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
, and some specific
results about the Galois groups of ℚ-polynomials with specific numbers of non-real roots.
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.
Instances For
If p
splits in F
then the p.gal
is trivial.
Instances For
Restrict from a superfield automorphism into a member of gal p
.
Instances For
The function taking rootSet p p.SplittingField
to rootSet p E
. This is actually a bijection,
see Polynomial.Gal.mapRoots_bijective
.
Instances For
The bijection between rootSet p p.SplittingField
and rootSet p E
.
Instances For
The action of gal p
on the roots of p
in E
.
Polynomial.Gal.restrict p E
is compatible with Polynomial.Gal.galAction p E
.
Polynomial.Gal.galAction
as a permutation representation
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.
Instances For
The Galois group of a product maps into the product of the Galois groups.
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.
Instances For
For a separable polynomial, its Galois group has cardinality
equal to the dimension of its splitting field over F
.
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).
An irreducible polynomial of prime degree with two non-real roots has full Galois group.
An irreducible polynomial of prime degree with 1-3 non-real roots has full Galois group.