Documentation

Mathlib.FieldTheory.SplittingField.Construction

Splitting fields #

In this file we prove the existence and uniqueness of splitting fields.

Main definitions #

Main statements #

Implementation details #

We construct a SplittingFieldAux without worrying about whether the instances satisfy nice definitional equalities. Then the actual SplittingField is defined to be a quotient of a MvPolynomial ring by the kernel of the obvious map into SplittingFieldAux. Because the actual SplittingField will be a quotient of a MvPolynomial, it has nice instances on it.

def Polynomial.factor {K : Type v} [Field K] (f : Polynomial K) :

Non-computably choose an irreducible factor from a polynomial.

Equations
Instances For

    See note [fact non-instances].

    theorem Polynomial.isCoprime_iff_aeval_ne_zero {K : Type v} [Field K] (f g : Polynomial K) :
    IsCoprime f g ∀ {A : Type v} [inst : CommRing A] [inst_1 : IsDomain A] [inst_2 : Algebra K A] (a : A), (aeval a) f 0 (aeval a) g 0

    Divide a polynomial f by X - C r where r is a root of f in a bigger field extension.

    Equations
    Instances For
      def Polynomial.SplittingFieldAuxAux (n : ) {K : Type u} [Field K] :
      Polynomial K(L : Type u) × (x : Field L) × Algebra K L

      Auxiliary construction to a splitting field of a polynomial, which removes n (arbitrarily-chosen) factors.

      It constructs the type, proves that is a field and algebra over the base field.

      Uses recursion on the degree.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def Polynomial.SplittingFieldAux (n : ) {K : Type u} [Field K] (f : Polynomial K) :

        Auxiliary construction to a splitting field of a polynomial, which removes n (arbitrarily-chosen) factors. It is the type constructed in SplittingFieldAuxAux.

        Equations
        Instances For

          A splitting field of a polynomial.

          Stacks Tag 09HV (The construction of the splitting field.)

          Equations
          Instances For
            Equations
            def Polynomial.SplittingField.lift {K : Type v} {L : Type w} [Field K] [Field L] (f : Polynomial K) [Algebra K L] (hb : Splits (algebraMap K L) f) :

            Embeds the splitting field into any other field that splits the polynomial.

            Equations
            Instances For

              Any splitting field is isomorphic to SplittingFieldAux f.

              Equations
              Instances For