Documentation

Mathlib.FieldTheory.PolynomialGaloisGroup

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 #

Main results #

Other results #

def Polynomial.Gal {F : Type u_1} [Field F] (p : Polynomial F) :
Type u_1

The Galois group of a polynomial.

Instances For
    theorem Polynomial.Gal.ext {F : Type u_1} [Field F] (p : Polynomial F) {σ : Polynomial.Gal p} {τ : Polynomial.Gal p} (h : ∀ (x : Polynomial.SplittingField p), x Polynomial.rootSet p (Polynomial.SplittingField p)σ x = τ x) :
    σ = τ

    If p splits in F then the p.gal is trivial.

    Instances For
      instance Polynomial.Gal.uniqueGalC {F : Type u_1} [Field F] (x : F) :
      Unique (Polynomial.Gal (Polynomial.C x))
      instance Polynomial.Gal.uniqueGalX {F : Type u_1} [Field F] :
      Unique (Polynomial.Gal Polynomial.X)
      instance Polynomial.Gal.uniqueGalXSubC {F : Type u_1} [Field F] (x : F) :
      Unique (Polynomial.Gal (Polynomial.X - Polynomial.C x))
      instance Polynomial.Gal.uniqueGalXPow {F : Type u_1} [Field F] (n : ) :
      Unique (Polynomial.Gal (Polynomial.X ^ n))
      def Polynomial.Gal.restrict {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Polynomial.Splits (algebraMap F E) p)] :

      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
            instance Polynomial.Gal.smul {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Polynomial.Splits (algebraMap F E) p)] :
            theorem Polynomial.Gal.smul_def {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Polynomial.Splits (algebraMap F E) p)] (ϕ : Polynomial.Gal p) (x : ↑(Polynomial.rootSet p E)) :
            instance Polynomial.Gal.galAction {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Polynomial.Splits (algebraMap F E) p)] :

            The action of gal p on the roots of p in E.

            @[simp]
            theorem Polynomial.Gal.restrict_smul {F : Type u_1} [Field F] {p : Polynomial F} {E : Type u_2} [Field E] [Algebra F E] [Fact (Polynomial.Splits (algebraMap F E) p)] (ϕ : E ≃ₐ[F] E) (x : ↑(Polynomial.rootSet p E)) :
            ↑(↑(Polynomial.Gal.restrict p E) ϕ x) = ϕ x

            Polynomial.Gal.restrict p E is compatible with Polynomial.Gal.galAction p E.

            Polynomial.Gal.galAction as a permutation representation

            Instances For
              theorem Polynomial.Gal.galActionHom_restrict {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Polynomial.Splits (algebraMap F E) p)] (ϕ : E ≃ₐ[F] E) (x : ↑(Polynomial.rootSet p E)) :
              ↑(↑(↑(Polynomial.Gal.galActionHom p E) (↑(Polynomial.Gal.restrict p E) ϕ)) x) = ϕ x

              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
                theorem Polynomial.Gal.restrictDvd_def {F : Type u_1} [Field F] {p : Polynomial F} {q : Polynomial F} [Decidable (q = 0)] (hpq : p q) :

                The Galois group of a product maps into the product of the Galois groups.

                Instances For
                  theorem Polynomial.Gal.mul_splits_in_splittingField_of_mul {F : Type u_1} [Field F] {p₁ : Polynomial F} {q₁ : Polynomial F} {p₂ : Polynomial F} {q₂ : Polynomial F} (hq₁ : q₁ 0) (hq₂ : q₂ 0) (h₁ : Polynomial.Splits (algebraMap F (Polynomial.SplittingField q₁)) p₁) (h₂ : Polynomial.Splits (algebraMap F (Polynomial.SplittingField q₂)) p₂) :

                  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.