Documentation

Mathlib.FieldTheory.PurelyInseparable.PerfectClosure

Basic results about relative perfect closure #

This file contains basic results about relative perfect closures.

Main definitions #

Main results #

Tags #

separable degree, degree, separable closure, purely inseparable

def perfectClosure (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] :

The relative perfect closure of F in E, consists of the elements x of E such that there exists a natural number n such that x ^ (ringExpChar F) ^ n is contained in F, where ringExpChar F is the exponential characteristic of F. It is also the maximal purely inseparable subextension of E / F (le_perfectClosure_iff).

Stacks Tag 09HH

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem mem_perfectClosure_iff {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {x : E} :
    x perfectClosure F E ∃ (n : ), x ^ ringExpChar F ^ n (algebraMap F E).range
    theorem mem_perfectClosure_iff_pow_mem {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] (q : ) [ExpChar F q] {x : E} :
    x perfectClosure F E ∃ (n : ), x ^ q ^ n (algebraMap F E).range
    theorem mem_perfectClosure_iff_natSepDegree_eq_one {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {x : E} :

    An element is contained in the relative perfect closure if and only if its minimal polynomial has separable degree one.

    A field extension E / F is purely inseparable if and only if the relative perfect closure of F in E is equal to E.

    The relative perfect closure of F in E is purely inseparable over F.

    instance perfectClosure.isAlgebraic (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] :

    The relative perfect closure of F in E is algebraic over F.

    If E / F is separable, then the perfect closure of F in E is equal to F. Note that the converse is not necessarily true (see https://math.stackexchange.com/a/3009197) even when E / F is algebraic.

    theorem le_perfectClosure (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) [h : IsPurelyInseparable F L] :

    An intermediate field of E / F is contained in the relative perfect closure of F in E if it is purely inseparable over F.

    theorem le_perfectClosure_iff (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (L : IntermediateField F E) :

    An intermediate field of E / F is contained in the relative perfect closure of F in E if and only if it is purely inseparable over F.

    theorem map_mem_perfectClosure_iff {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {K : Type w} [Field K] [Algebra F K] (i : E →ₐ[F] K) {x : E} :

    If i is an F-algebra homomorphism from E to K, then i x is contained in perfectClosure F K if and only if x is contained in perfectClosure F E.

    theorem perfectClosure.comap_eq_of_algHom {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {K : Type w} [Field K] [Algebra F K] (i : E →ₐ[F] K) :

    If i is an F-algebra homomorphism from E to K, then the preimage of perfectClosure F K under the map i is equal to perfectClosure F E.

    theorem perfectClosure.map_le_of_algHom {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {K : Type w} [Field K] [Algebra F K] (i : E →ₐ[F] K) :

    If i is an F-algebra homomorphism from E to K, then the image of perfectClosure F E under the map i is contained in perfectClosure F K.

    theorem perfectClosure.map_eq_of_algEquiv {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {K : Type w} [Field K] [Algebra F K] (i : E ≃ₐ[F] K) :

    If i is an F-algebra isomorphism of E and K, then the image of perfectClosure F E under the map i is equal to in perfectClosure F K.

    def perfectClosure.algEquivOfAlgEquiv {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {K : Type w} [Field K] [Algebra F K] (i : E ≃ₐ[F] K) :

    If E and K are isomorphic as F-algebras, then perfectClosure F E and perfectClosure F K are also isomorphic as F-algebras.

    Equations
    Instances For
      def AlgEquiv.perfectClosure {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] {K : Type w} [Field K] [Algebra F K] (i : E ≃ₐ[F] K) :

      Alias of perfectClosure.algEquivOfAlgEquiv.


      If E and K are isomorphic as F-algebras, then perfectClosure F E and perfectClosure F K are also isomorphic as F-algebras.

      Equations
      Instances For
        instance perfectClosure.perfectRing (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (p : ) [ExpChar E p] [PerfectRing E p] :

        If E is a perfect field of exponential characteristic p, then the (relative) perfect closure perfectClosure F E is perfect.

        instance perfectClosure.perfectField (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] [PerfectField E] :

        If E is a perfect field, then the (relative) perfect closure perfectClosure F E is perfect.

        F⟮x⟯ / F is a purely inseparable extension if and only if the minimal polynomial of x has separable degree one.

        theorem IntermediateField.isPurelyInseparable_adjoin_simple_iff_pow_mem (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (q : ) [hF : ExpChar F q] {x : E} :
        IsPurelyInseparable F Fx ∃ (n : ), x ^ q ^ n (algebraMap F E).range

        If F is of exponential characteristic q, then F⟮x⟯ / F is a purely inseparable extension if and only if x ^ (q ^ n) is contained in F for some n : ℕ.

        theorem IntermediateField.isPurelyInseparable_adjoin_iff_pow_mem (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (q : ) [hF : ExpChar F q] {S : Set E} :
        IsPurelyInseparable F (adjoin F S) xS, ∃ (n : ), x ^ q ^ n (algebraMap F E).range

        If F is of exponential characteristic q, then F(S) / F is a purely inseparable extension if and only if for any x ∈ S, x ^ (q ^ n) is contained in F for some n : ℕ.

        instance IntermediateField.isPurelyInseparable_sup (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (L1 L2 : IntermediateField F E) [h1 : IsPurelyInseparable F L1] [h2 : IsPurelyInseparable F L2] :

        A compositum of two purely inseparable extensions is purely inseparable.

        instance IntermediateField.isPurelyInseparable_iSup (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] {ι : Sort u_1} {t : ιIntermediateField F E} [h : ∀ (i : ι), IsPurelyInseparable F (t i)] :
        IsPurelyInseparable F (⨆ (i : ι), t i)

        A compositum of purely inseparable extensions is purely inseparable.

        theorem IntermediateField.adjoin_eq_adjoin_pow_expChar_pow_of_isSeparable (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (S : Set E) [Algebra.IsSeparable F (adjoin F S)] (q : ) [ExpChar F q] (n : ) :
        adjoin F S = adjoin F ((fun (x : E) => x ^ q ^ n) '' S)

        If F is a field of exponential characteristic q, F(S) / F is separable, then F(S) = F(S ^ (q ^ n)) for any natural number n.

        theorem IntermediateField.adjoin_eq_adjoin_pow_expChar_pow_of_isSeparable' (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] [Algebra.IsSeparable F E] (S : Set E) (q : ) [ExpChar F q] (n : ) :
        adjoin F S = adjoin F ((fun (x : E) => x ^ q ^ n) '' S)

        If E / F is a separable field extension of exponential characteristic q, then F(S) = F(S ^ (q ^ n)) for any subset S of E and any natural number n.

        theorem IntermediateField.adjoin_eq_adjoin_pow_expChar_of_isSeparable (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] (S : Set E) [Algebra.IsSeparable F (adjoin F S)] (q : ) [ExpChar F q] :
        adjoin F S = adjoin F ((fun (x : E) => x ^ q) '' S)

        If F is a field of exponential characteristic q, F(S) / F is separable, then F(S) = F(S ^ q).

        theorem IntermediateField.adjoin_eq_adjoin_pow_expChar_of_isSeparable' (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] [Algebra.IsSeparable F E] (S : Set E) (q : ) [ExpChar F q] :
        adjoin F S = adjoin F ((fun (x : E) => x ^ q) '' S)

        If E / F is a separable field extension of exponential characteristic q, then F(S) = F(S ^ q) for any subset S of E.

        theorem IntermediateField.adjoin_simple_eq_adjoin_pow_expChar_pow_of_isSeparable (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] {a : E} (ha : IsSeparable F a) (q : ) [ExpChar F q] (n : ) :
        Fa = Fa ^ q ^ n

        If F is a field of exponential characteristic q, a : E is separable over F, then F⟮a⟯ = F⟮a ^ q ^ n⟯ for any natural number n.

        theorem IntermediateField.adjoin_simple_eq_adjoin_pow_expChar_pow_of_isSeparable' (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] [Algebra.IsSeparable F E] (a : E) (q : ) [ExpChar F q] (n : ) :
        Fa = Fa ^ q ^ n

        If E / F is a separable field extension of exponential characteristic q, then F⟮a⟯ = F⟮a ^ q ^ n⟯ for any subset a : E and any natural number n.

        theorem IntermediateField.adjoin_simple_eq_adjoin_pow_expChar_of_isSeparable (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] {a : E} (ha : IsSeparable F a) (q : ) [ExpChar F q] :
        Fa = Fa ^ q

        If F is a field of exponential characteristic q, a : E is separable over F, then F⟮a⟯ = F⟮a ^ q⟯.

        theorem IntermediateField.adjoin_simple_eq_adjoin_pow_expChar_of_isSeparable' (F : Type u) (E : Type v) [Field F] [Field E] [Algebra F E] [Algebra.IsSeparable F E] (a : E) (q : ) [ExpChar F q] :
        Fa = Fa ^ q

        If E / F is a separable field extension of exponential characteristic q, then F⟮a⟯ = F⟮a ^ q⟯ for any a : E.

        theorem Field.span_map_pow_expChar_pow_eq_top_of_isSeparable {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] (q n : ) [hF : ExpChar F q] {ι : Type u_1} {v : ιE} [Algebra.IsSeparable F E] (h : Submodule.span F (Set.range v) = ) :
        Submodule.span F (Set.range fun (x : ι) => v x ^ q ^ n) =

        If E / F is a separable extension of exponential characteristic q, if { u_i } is a family of elements of E which F-linearly spans E, then { u_i ^ (q ^ n) } also F-linearly spans E for any natural number n.

        theorem LinearIndependent.map_pow_expChar_pow_of_isSeparable {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] (q n : ) [hF : ExpChar F q] {ι : Type u_1} {v : ιE} [Algebra.IsSeparable F E] (h : LinearIndependent F v) :
        LinearIndependent F fun (x : ι) => v x ^ q ^ n

        If E / F is a separable extension of exponential characteristic q, if { u_i } is a family of elements of E which is F-linearly independent, then { u_i ^ (q ^ n) } is also F-linearly independent for any natural number n.

        theorem LinearIndependent.map_pow_expChar_pow_of_isSeparable' {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] (q n : ) [hF : ExpChar F q] {ι : Type u_1} {v : ιE} (hsep : ∀ (i : ι), IsSeparable F (v i)) (h : LinearIndependent F v) :
        LinearIndependent F fun (x : ι) => v x ^ q ^ n

        If E / F is a field extension of exponential characteristic q, if { u_i } is a family of separable elements of E which is F-linearly independent, then { u_i ^ (q ^ n) } is also F-linearly independent for any natural number n.

        def Basis.mapPowExpCharPowOfIsSeparable {F : Type u} {E : Type v} [Field F] [Field E] [Algebra F E] (q n : ) [hF : ExpChar F q] {ι : Type u_1} [Algebra.IsSeparable F E] (b : Basis ι F E) :
        Basis ι F E

        If E / F is a separable extension of exponential characteristic q, if { u_i } is an F-basis of E, then { u_i ^ (q ^ n) } is also an F-basis of E for any natural number n.

        Equations
        Instances For

          If E / F is a separable extension, E is perfect, then F is also prefect.

          If E is an algebraic closure of F, then F is perfect if and only if E / F is separable.