Skip to content

Commit

Permalink
feat(algebra/group): add units.map and prove that it is a group hom
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Sep 27, 2018
1 parent a770ee5 commit bb97073
Showing 1 changed file with 13 additions and 0 deletions.
13 changes: 13 additions & 0 deletions algebra/group.lean
Expand Up @@ -696,3 +696,16 @@ calc f (a - b) = f (a + -b) : rfl
... = f a - f b : by simp[neg f]

end is_add_group_hom

namespace units
variables [monoid α] [monoid β] (f : α → β) [is_monoid_hom f]

definition map : units α → units β :=
λ u, ⟨f u.val, f u.inv,
by rw [← is_monoid_hom.map_mul f, u.val_inv, is_monoid_hom.map_one f],
by rw [← is_monoid_hom.map_mul f, u.inv_val, is_monoid_hom.map_one f] ⟩

instance : is_group_hom (units.map f) :=
⟨λ a b, by ext; exact is_monoid_hom.map_mul f ⟩

end units

0 comments on commit bb97073

Please sign in to comment.