Examples of divided power structures #
In this file we show that, for certain choices of a commutative (semi)ring A
and an ideal I
of
A
, the family of maps ℕ → A → A
given by fun n x ↦ x^n/n!
is a divided power structure on I
.
Main Definitions #
DividedPowers.OfInvertibleFactorial.dpow
: the family of functionsℕ → A → A
given byx^n/n!
.DividedPowers.OfInvertibleFactorial.dividedPowers
: the divided power structure onI
given byfun x n ↦ x^n/n!
, assuming that there exists a natural numbern
such thatf (n-1)!
is invertible inA
andI^n = 0
.DividedPowers.OfSquareZero.dividedPowers
: given an idealI
such thatI^2 =0
, this is the divided power structure onI
given byfun x n ↦ x^n/n!
.DividedPowers.CharP.dividedPowers
: ifA
is a commutative ring of prime characteristicp
andI
is an ideal such thatI^p = 0
, , this is the divided power structure onI
given byfun x n ↦ x^n/n!
.DividedPowers.RatAlgebra.dividedPowers
: ifI
is any ideal in aℚ
-algebra, this is the divided power structure onI
given byfun x n ↦ x^n/n!
.
Main Results #
DividedPowers.RatAlgebra.dividedPowers_unique
: there are no other divided power structures on an ideal of aℚ
-algebra.
References #
The family of functions ℕ → A → A
given by x^n/n!
.
Equations
- DividedPowers.OfInvertibleFactorial.dpow I m x = if x ∈ I then Ring.inverse ↑m.factorial * x ^ m else 0
Instances For
If (n-1)!
is invertible in A
and I^n = 0
, then I
admits a divided power structure.
Proposition 1.2.7 of [B74], part (ii).
Equations
- One or more equations did not get rendered due to their size.
Instances For
If I^2 = 0
, then I
admits a divided power structure.
Equations
Instances For
If A
is a commutative ring of prime characteristic p
and I
is an ideal such that
I^p = 0
, then I
admits a divided power structure.
Equations
Instances For
If A
is a commutative ring of prime characteristic p
and I
is an ideal such that
I^p = 0
, then I
admits a divided power structure.
Equations
Instances For
The family ℕ → R → R
given by dpow n x = x ^ n / n!
.
Instances For
If I
is an ideal in a ℚ
-algebra A
, then I
admits a unique divided power structure,
given by dpow n x = x ^ n / n!
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If I
is an ideal in a ℚ
-algebra A
, then the divided power structure on I
given by
dpow n x = x ^ n / n!
is the only possible one.
There are no other divided power structures on an ideal of a ℚ
-algebra.