The Schur-Zassenhaus Theorem #
In this file we prove the Schur-Zassenhaus theorem.
Main results #
exists_right_complement'_of_coprime
: The Schur-Zassenhaus theorem: IfH : subgroup G
is normal and has order coprime to its index, then there exists a subgroupK
which is a (right) complement ofH
.exists_left_complement'_of_coprime
The Schur-Zassenhaus theorem: IfH : subgroup G
is normal and has order coprime to its index, then there exists a subgroupK
which is a (left) complement ofH
.
Equations
- add_subgroup.left_transversals.add_action = {to_has_vadd := {vadd := λ (g : G) (T : ↥(add_subgroup.left_transversals ↑H)), ⟨g +l ↑T, _⟩}, zero_vadd := _, add_vadd := _}
Equations
- subgroup.left_transversals.mul_action = {to_has_scalar := {smul := λ (g : G) (T : ↥(subgroup.left_transversals ↑H)), ⟨g *l ↑T, _⟩}, one_smul := _, mul_smul := _}
The difference of two left transversals
Equations
- add_subgroup.diff α β = let α' : quotient (quotient_add_group.left_rel H) ≃ ↥(α.val) := (equiv.of_bijective (set.restrict quotient.mk' α.val) _).symm, β' : quotient (quotient_add_group.left_rel H) ≃ ↥(β.val) := (equiv.of_bijective (set.restrict quotient.mk' β.val) _).symm in ∑ (q : G ⧸ H), ⟨↑(⇑α' q) + -↑(⇑β' q), _⟩
The difference of two left transversals
Equations
- subgroup.diff α β = let α' : quotient (quotient_group.left_rel H) ≃ ↥(α.val) := (equiv.of_bijective (set.restrict quotient.mk' α.val) _).symm, β' : quotient (quotient_group.left_rel H) ≃ ↥(β.val) := (equiv.of_bijective (set.restrict quotient.mk' β.val) _).symm in ∏ (q : G ⧸ H), ⟨(↑(⇑α' q)) * (↑(⇑β' q))⁻¹, _⟩
Equations
- H.setoid_diff = {r := λ (α β : ↥(subgroup.left_transversals ↑H)), subgroup.diff α β = 1, iseqv := _}
The quotient of the transversals of an abelian normal N
by the diff
relation
Equations
Equations
Equations
- subgroup.quotient_diff.mul_action = {to_has_scalar := {smul := λ (g : G), quotient.map (λ (α : ↥(subgroup.left_transversals ↑H)), g • α) _}, one_smul := _, mul_smul := _}
Proof of the Schur-Zassenhaus theorem #
In this section, we prove the Schur-Zassenhaus theorem.
The proof is by contradiction. We assume that G
is a minimal counterexample to the theorem.
We will arrive at a contradiction via the following steps:
- step 0:
N
(the normal Hall subgroup) is nontrivial. - step 1: If
K
is a subgroup ofG
withK ⊔ N = ⊤
, thenK = ⊤
. - step 2:
N
is a minimal normal subgroup, phrased in terms of subgroups ofG
. - step 3:
N
is a minimal normal subgroup, phrased in terms of subgroups ofN
. - step 4:
p
(min_fact (fintype.card N)
) is prime (follows from step0). - step 5:
P
(a Sylowp
-subgroup ofN
) is nontrivial. - step 6:
N
is ap
-group (applies step 1 to the normalizer ofP
inG
). - step 7:
N
is abelian (applies step 3 to the center ofN
).
Do not use this lemma: It is made obsolete by exists_right_complement'_of_coprime
Schur-Zassenhaus for normal subgroups:
If H : subgroup G
is normal, and has order coprime to its index, then there exists a
subgroup K
which is a (right) complement of H
.
Schur-Zassenhaus for normal subgroups:
If H : subgroup G
is normal, and has order coprime to its index, then there exists a
subgroup K
which is a (right) complement of H
.
Schur-Zassenhaus for normal subgroups:
If H : subgroup G
is normal, and has order coprime to its index, then there exists a
subgroup K
which is a (left) complement of H
.
Schur-Zassenhaus for normal subgroups:
If H : subgroup G
is normal, and has order coprime to its index, then there exists a
subgroup K
which is a (left) complement of H
.