Documentation

Mathlib.GroupTheory.SpecificGroups.Alternating.KleinFour

The Klein Four subgroup of an alternating group on 4 letters #

Let α be a finite type such that Nat.card α = 4.

Main results #

Remark on implementation #

We start from alternatingGroup.kleinFour α as given by its definition. We first prove that it is equal to any 2-sylow subgroup: the elements of such a sylow subgroup S have order a power of 2, and this implies that their cycle type is () or (2,2). Since there are exactly 4 elements of that cycle type, we conclude that alternatingGroup.kleinFour α = S. Since all 2-sylow subgroups are conjugate, we conclude that there is only one 2-sylow subgroup and that it is normal, and then characteristic.

TODO : #

Prove alternatingGroup.kleinFour α = commutator (alternatingGroup α) without any assumption on Nat.card α.

The subgroup of alternatingGroup α generated by permutations of cycle type (2, 2).

When Nat.card α = 4, it will effectively be of Klein Four type.

Equations
Instances For
    theorem alternatingGroup.mem_kleinFour_of_order_two_pow {α : Type u_1} [DecidableEq α] [Fintype α] (hα4 : Nat.card α = 4) {g : Equiv.Perm α} (hg0 : g alternatingGroup α) {n : } (hg : orderOf g 2 ^ n) :
    theorem alternatingGroup.card_two_sylow_of_card_eq_four {α : Type u_1} [DecidableEq α] [Fintype α] (hα4 : Nat.card α = 4) (S : Sylow 2 (alternatingGroup α)) :
    Nat.card S = 4
    theorem alternatingGroup.coe_two_sylow_of_card_eq_four {α : Type u_1} [DecidableEq α] [Fintype α] (hα4 : Nat.card α = 4) (S : Sylow 2 (alternatingGroup α)) :
    S = {1} {g : (alternatingGroup α) | (↑g).cycleType = {2, 2}}
    theorem alternatingGroup.coe_kleinFour_of_card_eq_four {α : Type u_1} [DecidableEq α] [Fintype α] (hα4 : Nat.card α = 4) :
    (kleinFour α) = {1} {g : (alternatingGroup α) | (↑g).cycleType = {2, 2}}