Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): If H is commutative, then `H ≤ H…
Browse files Browse the repository at this point in the history
….centralizer` (#16718)

If `H` is commutative, then `H ≤ H.centralizer`.
  • Loading branch information
tb65536 committed Oct 1, 2022
1 parent 567220c commit d638c7f
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/group_theory/subgroup/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1859,6 +1859,12 @@ end⟩⟩
(H.subgroup_of K).is_commutative :=
H.comap_injective_is_commutative subtype.coe_injective

@[to_additive] lemma le_centralizer_iff_is_commutative : K ≤ K.centralizer ↔ K.is_commutative :=
⟨λ h, ⟨⟨λ x y, subtype.ext (h y.2 x x.2)⟩⟩, λ h x hx y hy, congr_arg coe (h.1.1 ⟨y, hy⟩ ⟨x, hx⟩)⟩

@[to_additive] lemma le_centralizer [h : H.is_commutative] : H ≤ H.centralizer :=
le_centralizer_iff_is_commutative.mpr h

end subgroup

namespace group
Expand Down

0 comments on commit d638c7f

Please sign in to comment.