Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): Centralizer of closure is intersec…
Browse files Browse the repository at this point in the history
…tion of centralizers (#16394)

This PR adds some more API for `subgroup.centralizer` and proves that the centralizer of a closure is the intersection of the centralizers.
  • Loading branch information
tb65536 committed Sep 7, 2022
1 parent 6211945 commit 13c6c43
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/group_theory/subgroup/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1787,6 +1787,8 @@ def centralizer : subgroup G :=
inv_mem' := λ g, set.inv_mem_centralizer,
.. submonoid.centralizer ↑H }

variables {H}

@[to_additive] lemma mem_centralizer_iff {g : G} : g ∈ H.centralizer ↔ ∀ h ∈ H, h * g = g * h :=
iff.rfl

Expand All @@ -1797,6 +1799,12 @@ by simp only [mem_centralizer_iff, mul_inv_eq_iff_eq_mul, one_mul]
@[to_additive] lemma centralizer_top : centralizer ⊤ = center G :=
set_like.ext' (set.centralizer_univ G)

@[to_additive] lemma le_centralizer_iff : H ≤ K.centralizer ↔ K ≤ H.centralizer :=
⟨λ h x hx y hy, (h hy x hx).symm, λ h x hx y hy, (h hy x hx).symm⟩

@[to_additive] lemma centralizer_le (h : H ≤ K) : centralizer K ≤ centralizer H :=
submonoid.centralizer_le h

@[to_additive] instance subgroup.centralizer.characteristic [hH : H.characteristic] :
H.centralizer.characteristic :=
begin
Expand Down Expand Up @@ -2699,6 +2707,12 @@ by rw [eq_bot_iff, zpowers_le, mem_bot]
subgroup.zpowers (1 : G) = ⊥ :=
subgroup.zpowers_eq_bot.mpr rfl

@[to_additive] lemma centralizer_closure (S : set G) :
(closure S).centralizer = ⨅ g ∈ S, (zpowers g).centralizer :=
le_antisymm (le_infi $ λ g, le_infi $ λ hg, centralizer_le $ zpowers_le.2 $ subset_closure hg)
$ le_centralizer_iff.1 $ (closure_le _).2
$ λ g, set_like.mem_coe.2 ∘ zpowers_le.1 ∘ le_centralizer_iff.1 ∘ infi_le_of_le g ∘ infi_le _

end subgroup

namespace monoid_hom
Expand Down

0 comments on commit 13c6c43

Please sign in to comment.