Skip to content

Commit

Permalink
feat(group_theory/group_action/conj_act): A characteristic subgroup o…
Browse files Browse the repository at this point in the history
…f a normal subgroup is normal (#9992)

Uses `mul_aut.conj_normal` to prove an instance stating that a characteristic subgroup of a normal subgroup is normal.
  • Loading branch information
tb65536 committed Oct 27, 2021
1 parent c529711 commit eaec1da
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/group_theory/group_action/conj_act.lean
Expand Up @@ -144,4 +144,11 @@ lemma _root_.mul_aut.conj_normal_coe {H : subgroup G} [H.normal] {h : H} :
mul_aut.conj_normal ↑h = mul_aut.conj h :=
mul_equiv.ext (λ x, rfl)

instance normal_of_characteristic_of_normal {H : subgroup G} [hH : H.normal]
{K : subgroup H} [h : K.characteristic] : (K.map H.subtype).normal :=
⟨λ a ha b, by
{ obtain ⟨a, ha, rfl⟩ := ha,
exact K.apply_coe_mem_map H.subtype
⟨_, ((set_like.ext_iff.mp (h.fixed (mul_aut.conj_normal b)) a).mpr ha)⟩ }⟩

end conj_act

0 comments on commit eaec1da

Please sign in to comment.