Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit d638c7f

Browse files
committed
feat(group_theory/subgroup/basic): If H is commutative, then H ≤ H.centralizer (#16718)
If `H` is commutative, then `H ≤ H.centralizer`.
1 parent 567220c commit d638c7f

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

src/group_theory/subgroup/basic.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1859,6 +1859,12 @@ end⟩⟩
18591859
(H.subgroup_of K).is_commutative :=
18601860
H.comap_injective_is_commutative subtype.coe_injective
18611861

1862+
@[to_additive] lemma le_centralizer_iff_is_commutative : K ≤ K.centralizer ↔ K.is_commutative :=
1863+
⟨λ 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⟩)⟩
1864+
1865+
@[to_additive] lemma le_centralizer [h : H.is_commutative] : H ≤ H.centralizer :=
1866+
le_centralizer_iff_is_commutative.mpr h
1867+
18621868
end subgroup
18631869

18641870
namespace group

0 commit comments

Comments
 (0)