Skip to content

Commit

Permalink
refactor(group_theory/commutator): Generalize map_commutator_element (
Browse files Browse the repository at this point in the history
#12555)

This PR generalizes `map_commutator_element` from `monoid_hom_class F G G` to `monoid_hom_class F G G'`.
  • Loading branch information
tb65536 committed Mar 10, 2022
1 parent 24e3b5f commit 1e560a6
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/group_theory/commutator.lean
Expand Up @@ -21,12 +21,12 @@ is the subgroup of `G` generated by the commutators `h₁ * h₂ * h₁⁻¹ * h
* `⁅H₁, H₂⁆` : the commutator of the subgroups `H₁` and `H₂`.
-/

variables {G G' F : Type*} [group G] [group G'] [monoid_hom_class F G G] (f : F) (g₁ g₂ g₃ : G)
variables {G G' F : Type*} [group G] [group G'] [monoid_hom_class F G G'] (f : F) (g₁ g₂ g₃ : G)

@[simp] lemma commutator_element_inv : ⁅g₁, g₂⁆⁻¹ = ⁅g₂, g₁⁆ :=
by simp_rw [commutator_element_def, mul_inv_rev, inv_inv, mul_assoc]

lemma map_commutator_element : f ⁅g₁, g₂⁆ = ⁅f g₁, f g₂⁆ :=
lemma map_commutator_element : (f ⁅g₁, g₂⁆ : G') = ⁅f g₁, f g₂⁆ :=
by simp_rw [commutator_element_def, map_mul f, map_inv f]

lemma conjugate_commutator_element : g₃ * ⁅g₁, g₂⁆ * g₃⁻¹ = ⁅g₃ * g₁ * g₃⁻¹, g₃ * g₂ * g₃⁻¹⁆ :=
Expand Down

0 comments on commit 1e560a6

Please sign in to comment.