Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): The centralizer of a characteristi…
Browse files Browse the repository at this point in the history
…c subgroup is characteristic (#13230)

This PR proves that the centralizer of a characteristic subgroup is characteristic.
  • Loading branch information
tb65536 committed Apr 8, 2022
1 parent 95ebbad commit e85dc17
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -1790,6 +1790,14 @@ 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] instance subgroup.centralizer.characteristic [hH : H.characteristic] :
H.centralizer.characteristic :=
begin
refine subgroup.characteristic_iff_comap_le.mpr (λ ϕ g hg h hh, ϕ.injective _),
rw [map_mul, map_mul],
exact hg (ϕ h) (subgroup.characteristic_iff_le_comap.mp hH ϕ hh),
end

end centralizer

/-- Commutivity of a subgroup -/
Expand Down

0 comments on commit e85dc17

Please sign in to comment.