Divided power morphisms #
Let A
and B
be commutative (semi)rings, let I
be an ideal of A
and let J
be an ideal of
B
. Given divided power structures on I
and J
, a ring morphism A →+* B
is a divided
power morphism if it is compatible with these divided power structures.
Main definitions #
DividedPowers.IsDPMorphism
: given divided power structures on theA
-idealI
and theB
-idealJ
, a ring morphismA →+* B
is a divided power morphism if it is compatible with these divided power structures.DividedPowers.DPMorphism
: a bundled version ofIsDPMorphism
.DividedPowers.ideal_from_ringHom
: given a ring homomorphismA →+* B
and idealsI ⊆ A
andJ ⊆ B
such thatI.map f ≤ J
, this is theA
-ideal on whichf (hI.dpow n x) = hJ.dpow n (f x)
.DividedPowers.DPMorphism.fromGens
: theDPMorphism
induced by a ring morphism, given that divided powers are compatible on a generating set.
Main results #
DividedPowers.dpow_eq_from_gens
: if two divided power structures on an idealI
agree on a generating set, then they are equal.
Implementation remarks #
We provided both a bundled and an unbundled definition of divided power morphisms. For developing
the basic theory, the unbundled version IsDPMorphism
is more convenient. However, we anticipate
that the bundled version DPMorphism
will be better for the development of crystalline
cohomology.
References #
Given divided power structures on the A
-ideal I
and the B
-ideal J
, a ring morphism
A → B
is a divided power morphism if it is compatible with these divided power structures.
Instances For
A bundled divided power morphism between rings endowed with divided power structures.
- toFun : A → B
Instances For
Equations
- DividedPowers.DPMorphism.instFunLike hI hJ = { coe := fun (h : hI.DPMorphism hJ) => ⇑h.toRingHom, coe_injective' := ⋯ }
Equations
- DividedPowers.DPMorphism.coe_ringHom hI hJ = { coe := DividedPowers.DPMorphism.toRingHom }
A constructor for DPMorphism
from a ring homomorphism f : A →+* B
satisfying
IsDPMorphism hI hJ f
.
Equations
- DividedPowers.DPMorphism.mk' hf = { toRingHom := f, ideal_comp := ⋯, dpow_comp := ⋯ }
Instances For
Given a ring homomorphism A → B
and ideals I ⊆ A
and J ⊆ B
such that I.map f ≤ J
,
this is the A
-ideal on which f (hI.dpow n x) = hJ.dpow n (f x)
.
See N. Roby, Les algèbres à puissances dividées (Proposition 2).
Equations
Instances For
The DPMorphism
induced by a ring morphism, given that divided powers are compatible on a
generating set.
See N. Roby, Les algèbres à puissances dividées (Proposition 3).
Equations
- DividedPowers.DPMorphism.fromGens hI hJ hS hf h = { toRingHom := f, ideal_comp := hf, dpow_comp := ⋯ }
Instances For
The identity map as a DPMorphism
.
Equations
- DividedPowers.DPMorphism.id hI = { toRingHom := RingHom.id A, ideal_comp := ⋯, dpow_comp := ⋯ }
Instances For
Equations
- DividedPowers.DPMorphism.instInhabited hI = { default := DividedPowers.DPMorphism.id hI }
The composition of two divided power morphisms as a DPMorphism
.
Equations
Instances For
If two divided power structures on the ideal I
agree on a generating set, then they are
equal.
See N. Roby, Les algèbres à puissances dividées (Corollary to Proposition 3).