Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): add commute_of_normal_of_disjoint (#…
Browse files Browse the repository at this point in the history
…11751)




Co-authored-by: Johan Commelin <johan@commelin.net>
  • Loading branch information
nomeata and jcommelin committed Feb 2, 2022
1 parent a6d70aa commit 664b5be
Showing 1 changed file with 16 additions and 0 deletions.
16 changes: 16 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -2475,6 +2475,22 @@ begin
rwa [mul_assoc, mul_assoc, mul_right_inv, mul_one] at this,
end

/-- Elements of disjoint, normal subgroups commute -/
@[to_additive] lemma commute_of_normal_of_disjoint
(H₁ H₂ : subgroup G) (hH₁ : H₁.normal) (hH₂ : H₂.normal) (hdis : disjoint H₁ H₂)
(x y : G) (hx : x ∈ H₁) (hy : y ∈ H₂) :
commute x y :=
begin
suffices : x * y * x⁻¹ * y⁻¹ = 1,
{ show x * y = y * x, by { rw [mul_assoc, mul_eq_one_iff_eq_inv] at this, simpa } },
apply hdis, split,
{ suffices : x * (y * x⁻¹ * y⁻¹) ∈ H₁, by simpa [mul_assoc],
exact H₁.mul_mem hx (hH₁.conj_mem _ (H₁.inv_mem hx) _) },
{ show x * y * x⁻¹ * y⁻¹ ∈ H₂,
apply H₂.mul_mem _ (H₂.inv_mem hy),
apply (hH₂.conj_mem _ hy), }
end

end subgroup_normal

end subgroup
Expand Down

0 comments on commit 664b5be

Please sign in to comment.