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.

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.

Equations
Instances For
    theorem Polynomial.Gal.ext {F : Type u_1} [Field F] (p : Polynomial F) {σ τ : p.Gal} (h : ∀ (x : p.SplittingField), Membership.mem (p.rootSet p.SplittingField) xEq (DFunLike.coe σ x) (DFunLike.coe τ x)) :
    Eq σ τ
    theorem Polynomial.Gal.ext_iff {F : Type u_1} [Field F] {p : Polynomial F} {σ τ : p.Gal} :
    Iff (Eq σ τ) (∀ (x : p.SplittingField), Membership.mem (p.rootSet p.SplittingField) xEq (DFunLike.coe σ x) (DFunLike.coe τ x))

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

    Equations
    Instances For
      def Polynomial.Gal.restrict {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] :

      Restrict from a superfield automorphism into a member of gal p.

      Equations
      Instances For
        def Polynomial.Gal.mapRoots {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] :

        The function taking rootSet p p.SplittingField to rootSet p E. This is actually a bijection, see Polynomial.Gal.mapRoots_bijective.

        Equations
        Instances For
          theorem Polynomial.Gal.mapRoots_bijective {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [h : Fact (Splits (algebraMap F E) p)] :
          def Polynomial.Gal.rootsEquivRoots {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] :

          The bijection between rootSet p p.SplittingField and rootSet p E.

          Equations
          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def Polynomial.Gal.smul {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] :
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                theorem Polynomial.Gal.smul_def {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] (ϕ : p.Gal) (x : (p.rootSet E).Elem) :
                def Polynomial.Gal.galAction {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] :

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

                Equations
                Instances For
                  theorem Polynomial.Gal.restrict_smul {F : Type u_1} [Field F] {p : Polynomial F} {E : Type u_2} [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] (ϕ : AlgEquiv F E E) (x : (p.rootSet E).Elem) :

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

                  def Polynomial.Gal.galActionHom {F : Type u_1} [Field F] (p : Polynomial F) (E : Type u_2) [Field E] [Algebra F E] [Fact (Splits (algebraMap F E) p)] :

                  Polynomial.Gal.galAction as a permutation representation

                  Equations
                  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 (Splits (algebraMap F E) p)] (ϕ : AlgEquiv F E E) (x : (p.rootSet E).Elem) :

                    gal p embeds as a subgroup of permutations of the roots of p in E.

                    def Polynomial.Gal.restrictDvd {F : Type u_1} [Field F] {p q : Polynomial F} (hpq : Dvd.dvd p q) :

                    Polynomial.Gal.restrict, when both fields are splitting fields of polynomials.

                    Equations
                    Instances For
                      theorem Polynomial.Gal.restrictDvd_def {F : Type u_1} [Field F] {p q : Polynomial F} [Decidable (Eq q 0)] (hpq : Dvd.dvd p q) :
                      Eq (restrictDvd hpq) (if hq : Eq q 0 then 1 else restrict p q.SplittingField)

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

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

                        p splits in the splitting field of p ∘ q, for q non-constant.

                        def Polynomial.Gal.restrictComp {F : Type u_1} [Field F] (p q : Polynomial F) (hq : Ne q.natDegree 0) :

                        Polynomial.Gal.restrict for the composition of polynomials.

                        Equations
                        Instances For

                          For a separable polynomial, its Galois group has cardinality equal to the dimension of its splitting field over F.