Documentation

Mathlib.FieldTheory.IsAlgClosed.AlgebraicClosure

Algebraic Closure #

In this file we construct the algebraic closure of a field

Main Definitions #

Tags #

algebraic closure, algebraically closed

@[reducible, inline]

The subtype of monic irreducible polynomials

Equations
Instances For

    Sends a monic irreducible polynomial f to f(x_f) where x_f is a formal indeterminate.

    Equations
    Instances For

      The span of f(x_f) across monic irreducible polynomials f where x_f is an indeterminate.

      Equations
      Instances For

        Given a finset of monic irreducible polynomials, construct an algebra homomorphism to the splitting field of the product of the polynomials sending each indeterminate x_f represented by the polynomial f in the finset to a root of f.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          A random maximal ideal that contains spanEval k

          Equations
          Instances For
            def AlgebraicClosure (k : Type u) [Field k] :

            The canonical algebraic closure of a field, the direct limit of adding roots to the field for each polynomial over the field.

            Stacks Tag 09GT

            Equations
            Instances For
              instance AlgebraicClosure.instIsScalarTower (k : Type u) [Field k] {R : Type u_1} {S : Type u_2} [CommSemiring R] [CommSemiring S] [Algebra R S] [Algebra S k] [Algebra R k] [IsScalarTower R S k] :
              Equations