Galois Groups of Polynomials #
In this file, we introduce the Galois group of a polynomial p
over a field F
,
defined as the automorphism group of its splitting field. We also provide
some results about some extension E
above p.SplittingField
.
Main definitions #
Polynomial.Gal p
: the Galois group of a polynomial p.Polynomial.Gal.restrict p E
: the restriction homomorphism(E ≃ₐ[F] E) → gal p
.Polynomial.Gal.galAction p E
: the action ofgal p
on the roots ofp
inE
.
Main results #
Polynomial.Gal.restrict_smul
:restrict p E
is compatible withgal_action p E
.Polynomial.Gal.galActionHom_injective
:gal p
acting on the roots ofp
inE
is faithful.Polynomial.Gal.restrictProd_injective
:gal (p * q)
embeds as a subgroup ofgal p × gal q
.Polynomial.Gal.card_of_separable
: For a separable polynomial, its Galois group has cardinality equal to the dimension of its splitting field overF
.Polynomial.Gal.galActionHom_bijective_of_prime_degree
: An irreducible polynomial of prime degree with two non-real roots has full Galois group.
Other results #
Polynomial.Gal.card_complex_roots_eq_card_real_add_card_not_gal_inv
: The number of complex roots equals the number of real roots plus the number of roots not fixed by complex conjugation (i.e. with some imaginary component).
The Galois group of a polynomial.
Equations
- Eq p.Gal (AlgEquiv F p.SplittingField p.SplittingField)
Instances For
Equations
- Eq (Polynomial.Gal.instGroup p) (inferInstanceAs (Group (AlgEquiv F p.SplittingField p.SplittingField)))
Instances For
Equations
- Eq (Polynomial.Gal.instFintype p) (inferInstanceAs (Fintype (AlgEquiv F p.SplittingField p.SplittingField)))
Instances For
Equations
Instances For
Instances For
If p
splits in F
then the p.gal
is trivial.
Equations
- Eq (Polynomial.Gal.uniqueGalOfSplits p h) { default := 1, uniq := ⋯ }
Instances For
Equations
Instances For
Equations
Instances For
Equations
Instances For
Equations
Instances For
Instances For
Equations
Instances For
Equations
Instances For
Restrict from a superfield automorphism into a member of gal p
.
Equations
Instances For
The function taking rootSet p p.SplittingField
to rootSet p E
. This is actually a bijection,
see Polynomial.Gal.mapRoots_bijective
.
Equations
- Eq (Polynomial.Gal.mapRoots p E) (Set.MapsTo.restrict (DFunLike.coe (IsScalarTower.toAlgHom F p.SplittingField E)) (p.rootSet p.SplittingField) (p.rootSet E) ⋯)
Instances For
The bijection between rootSet p p.SplittingField
and rootSet p E
.
Equations
- Eq (Polynomial.Gal.rootsEquivRoots p E) (Equiv.ofBijective (Polynomial.Gal.mapRoots p E) ⋯)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
The action of gal p
on the roots of p
in E
.
Equations
- Eq (Polynomial.Gal.galAction p E) { toSMul := Polynomial.Gal.smul p E, one_smul := ⋯, mul_smul := ⋯ }
Instances For
Polynomial.Gal.restrict p E
is compatible with Polynomial.Gal.galAction p E
.
Polynomial.Gal.galAction
as a permutation representation
Equations
- Eq (Polynomial.Gal.galActionHom p E) (MulAction.toPermHom p.Gal (p.rootSet E).Elem)
Instances For
gal p
embeds as a subgroup of permutations of the roots of p
in E
.
Polynomial.Gal.restrict
, when both fields are splitting fields of polynomials.
Equations
- Eq (Polynomial.Gal.restrictDvd hpq) (if hq : Eq q 0 then 1 else Polynomial.Gal.restrict p q.SplittingField)
Instances For
The Galois group of a product maps into the product of the Galois groups.
Equations
Instances For
Polynomial.Gal.restrictProd
is actually a subgroup embedding.
p
splits in the splitting field of p ∘ q
, for q
non-constant.
Polynomial.Gal.restrict
for the composition of polynomials.
Equations
- Eq (Polynomial.Gal.restrictComp p q hq) (Polynomial.Gal.restrict p (p.comp q).SplittingField)
Instances For
For a separable polynomial, its Galois group has cardinality
equal to the dimension of its splitting field over F
.