Skip to content

Commit

Permalink
feat(group_theory/commutator): Prove `commutator_eq_bot_iff_le_centra…
Browse files Browse the repository at this point in the history
…lizer` (#12598)

This lemma is needed for the three subgroups lemma.
  • Loading branch information
tb65536 committed Mar 12, 2022
1 parent b9ab27b commit 9456a74
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/group_theory/commutator.lean
Expand Up @@ -95,6 +95,14 @@ commutator_le.mpr (λ g₁ h₁ g₂ h₂,
lemma commutator_comm (H₁ H₂ : subgroup G) : ⁅H₁, H₂⁆ = ⁅H₂, H₁⁆ :=
le_antisymm (commutator_comm_le H₁ H₂) (commutator_comm_le H₂ H₁)

lemma commutator_eq_bot_iff_le_centralizer {H₁ H₂ : subgroup G} :
⁅H₁, H₂⁆ = ⊥ ↔ H₁ ≤ H₂.centralizer :=
begin
rw [eq_bot_iff, commutator_le],
refine forall_congr (λ p, forall_congr (λ hp, forall_congr (λ q, forall_congr (λ hq, _)))),
rw [mem_bot, commutator_element_eq_one_iff_mul_comm, eq_comm],
end

lemma commutator_le_right (H₁ H₂ : subgroup G) [h : normal H₂] : ⁅H₁, H₂⁆ ≤ H₂ :=
commutator_le.mpr (λ g₁ h₁ g₂ h₂, H₂.mul_mem (h.conj_mem g₂ h₂ g₁) (H₂.inv_mem h₂))

Expand Down

0 comments on commit 9456a74

Please sign in to comment.