IsPerfectClosure predicate #
This file contains IsPerfectClosure which asserts that L is a perfect closure of K under a
ring homomorphism i : K →+* L, as well as its basic properties.
Main definitions #
pNilradical: given a natural numberp, thep-nilradical of a ring is defined to be the nilradical ifp > 1(pNilradical_eq_nilradical), and defined to be the zero ideal ifp ≤ 1(pNilradical_eq_bot'). Equivalently, it is the ideal consisting of elementsxsuch thatx ^ p ^ n = 0for somen(mem_pNilradical).IsPRadical: a ring homomorphismi : K →+* Lof characteristicprings is calledp-radical, if or any elementxofLthere isn : ℕsuch thatx ^ (p ^ n)is contained inK, and the kernel ofiis contained in thep-nilradical ofK. A generalization of purely inseparable extension for fields.IsPerfectClosure: ifi : K →+* Lisp-radical ring homomorphism, then it makesLa perfect closure ofK, ifLis perfect.Our definition makes it synonymous to
IsPRadicalifPerfectRing L pis present. A caveat is that you need to write[PerfectRing L p] [IsPerfectClosure i p]. This is similar toPerfectRingwhich hasExpCharas a prerequisite.PerfectRing.lift: if ap-radical ring homomorphismK →+* Lis given,Mis a perfect ring, then any ring homomorphismK →+* Mcan be lifted toL →+* M. This is similar toIsAlgClosed.liftandIsSepClosed.lift.PerfectRing.liftEquiv:K →+* Mis one-to-one correspondence toL →+* M, given byPerfectRing.lift. This is a generalization toPerfectClosure.lift.IsPerfectClosure.equiv: perfect closures of a ring are isomorphic.
Main results #
IsPRadical.trans: composition ofp-radical ring homomorphisms is alsop-radical.PerfectClosure.isPRadical: the absolute perfect closurePerfectClosureis ap-radical extension over the base ring, in particular, it is a perfect closure of the base ring.IsPRadical.isPurelyInseparable,IsPurelyInseparable.isPRadical:p-radical and purely inseparable are equivalent for fields.The (relative) perfect closure
perfectClosureis a perfect closure (inferred fromIsPurelyInseparable.isPRadicalautomatically by Lean).
Tags #
perfect ring, perfect closure, purely inseparable
Given a natural number p, the p-nilradical of a ring is defined to be the
nilradical if p > 1 (pNilradical_eq_nilradical), and defined to be the zero ideal if p ≤ 1
(pNilradical_eq_bot'). Equivalently, it is the ideal consisting of elements x such that
x ^ p ^ n = 0 for some n (mem_pNilradical).
Equations
- pNilradical R p = if 1 < p then nilradical R else ⊥
Instances For
If i : K →+* L is a ring homomorphism of characteristic p rings, then it is called
p-radical if the following conditions are satisfied:
- For any element
xofLthere isn : ℕsuch thatx ^ (p ^ n)is contained inK. - The kernel of
iis contained in thep-nilradical ofK.
It is a generalization of purely inseparable extension for fields.
Instances
Composition of p-radical ring homomorphisms is also p-radical.
If i : K →+* L is a p-radical ring homomorphism, then it makes L a perfect closure
of K, if L is perfect.
In this case the kernel of i is equal to the p-nilradical of K
(see IsPerfectClosure.ker_eq).
Our definition makes it synonymous to IsPRadical if PerfectRing L p is present. A caveat is
that you need to write [PerfectRing L p] [IsPerfectClosure i p]. This is similar to
PerfectRing which has ExpChar as a prerequisite.
Equations
- IsPerfectClosure i p = IsPRadical i p
Instances For
If i : K →+* L is a ring homomorphism of exponential characteristic p rings, such that L
is perfect, then the p-nilradical of K is contained in the kernel of i.
If i : K →+* L and j : K →+* M are ring homomorphisms of characteristic p rings, such that
i is p-radical (in fact only the IsPRadical.pow_mem is required) and M is a perfect ring,
then one can define a map L → M which maps an element x of L to y ^ (p ^ -n) if
x ^ (p ^ n) is equal to some element y of K.
Equations
- PerfectRing.liftAux i j p x = (iterateFrobeniusEquiv M p (Classical.choose ⋯).1).symm (j (Classical.choose ⋯).2)
Instances For
If i : K →+* L is p-radical, then for any ring M of exponential charactistic p whose
p-nilradical is zero, the map (L →+* M) → (K →+* M) induced by i is injective.
If i : K →+* L is p-radical, then for any reduced ring M of exponential charactistic p,
the map (L →+* M) → (K →+* M) induced by i is injective.
A special case of IsPRadical.injective_comp_of_pNilradical_eq_bot
and a generalization of IsPurelyInseparable.injective_comp_algebraMap.
If i : K →+* L is p-radical, then for any perfect ring M of exponential charactistic p,
the map (L →+* M) → (K →+* M) induced by i is injective.
A special case of IsPRadical.injective_comp_of_pNilradical_eq_bot.
If i : K →+* L and j : K →+* M are ring homomorphisms of characteristic p rings, such that
i is p-radical, and M is a perfect ring, then PerfectRing.liftAux is well-defined.
If i : K →+* L and j : K →+* M are ring homomorphisms of characteristic p rings, such that
i is p-radical, and M is a perfect ring, then PerfectRing.liftAux
is a ring homomorphism. This is similar to IsAlgClosed.lift and IsSepClosed.lift.
Equations
- PerfectRing.lift i j p = { toFun := PerfectRing.liftAux i j p, map_one' := ⋯, map_mul' := ⋯, map_zero' := ⋯, map_add' := ⋯ }
Instances For
If i : K →+* L is a homomorphisms of characteristic p rings, such that
i is p-radical, and M is a perfect ring of characteristic p,
then K →+* M is one-to-one correspondence to
L →+* M, given by PerfectRing.lift. This is a generalization to PerfectClosure.lift.
Equations
- PerfectRing.liftEquiv M i p = { toFun := fun (j : K →+* M) => PerfectRing.lift i j p, invFun := fun (f : L →+* M) => f.comp i, left_inv := ⋯, right_inv := ⋯ }
Instances For
If L and M are both perfect closures of K, then there is a ring isomorphism L ≃+* M.
This is similar to IsAlgClosure.equiv and IsSepClosure.equiv.
Equations
- IsPerfectClosure.equiv i j p = { toFun := (↑↑(PerfectRing.lift i j p)).toFun, invFun := PerfectRing.liftAux j i p, left_inv := ⋯, right_inv := ⋯, map_mul' := ⋯, map_add' := ⋯ }
Instances For
The absolute perfect closure PerfectClosure is a p-radical extension over the base ring.
In particular, it is a perfect closure of the base ring, that is,
IsPerfectClosure (PerfectClosure.of K p) p.
If L / K is a p-radical field extension, then it is purely inseparable.
If L / K is a purely inseparable field extension, then it is p-radical. In particular, if
L is perfect, then the (relative) perfect closure perfectClosure K L is a perfect closure
of K, that is, IsPerfectClosure (algebraMap K (perfectClosure K L)) p.