Divided powers on ℤ_[p] #
Given a divided power algebra (B, J, δ)
and an injective ring morphism f : A →+* B
, if I
is
an A
-ideal such that I.map f = J
and such that for all n : ℕ
, x ∈ I
, the preimage of
hJ.dpow n (f x)
under f
belongs to I
, we get an induced divided power structure on I
.
We specialize this construction to the coercion map ℤ_[p] →+* ℚ_[p]
to get a divided power
structure on the ideal (p) ⊆ ℤ_[p]
. This divided power structure is given by the family of maps
fun n x ↦ x^n / n!
.
TODO: If K
is a p
-adic local field with ring of integers R
and uniformizer π
such that
p = u * π^e
for some unit u
, then the ideal (π) ⊆ R
has divided powers if and only if
e ≤ p - 1
.
Given a divided power algebra (B, J, δ)
and an injective ring morphism f : A →+* B
, if I
is an A
-ideal such that I.map f = J
and such that for all n : ℕ
, x ∈ I
, the preimage of
hJ.dpow n (f x)
under f
belongs to I
, this is the induced divided power structure on I
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The family ℕ → Ideal.span {(p : ℤ_[p])} → ℤ_[p]
given by dpow n x = x ^ n / n!
is a
divided power structure on the ℤ_[p]
-ideal (p)
.