Weierstrass preparation theorem for power series over a complete local ring #
In this file we define Weierstrass division, Weierstrass factorization, and prove Weierstrass preparation theorem.
We assume that a ring is adic complete with respect to some ideal.
If such ideal is a maximal ideal, then by isLocalRing_of_isAdicComplete_maximal
,
such ring has only one maximal ideal, and hence it is a complete local ring.
Main definitions #
PowerSeries.IsWeierstrassDivisionAt f g q r I
: letf
andg
be power series overA
,I
be an ideal ofA
, this is aProp
which asserts that a power seriesq
and a polynomialr
of degree< n
satisfyf = g * q + r
, wheren
is the order of the image ofg
in(A / I)⟦X⟧
(defined to be zero if such image is zero, in which case it's mathematically not considered).PowerSeries.IsWeierstrassDivision
: version ofPowerSeries.IsWeierstrassDivisionAt
for local rings with respect to its maximal ideal.PowerSeries.IsWeierstrassDivisorAt g I
: letg
be a power series overA
,I
be an ideal ofA
, this is aProp
which asserts that then
-th coefficient ofg
is a unit, wheren
is the order of the image ofg
in(A / I)⟦X⟧
(defined to be zero if such image is zero, in which case it's mathematically not considered).This property guarantees that if the
A
isI
-adic complete, theng
can be used as a divisor in Weierstrass division (PowerSeries.IsWeierstrassDivisorAt.isWeierstrassDivisionAt_div_mod
).PowerSeries.IsWeierstrassDivisor
: version ofPowerSeries.IsWeierstrassDivisorAt
for local rings with respect to its maximal ideal.PowerSeries.IsWeierstrassFactorizationAt g f h I
: for a power seriesg
overA
and an idealI
ofA
, this is aProp
which asserts thatf
is a distinguished polynomial atI
,h
is a formal power series overA
that is a unit and such thatg = f * h
.PowerSeries.IsWeierstrassFactorization
: version ofPowerSeries.IsWeierstrassFactorizationAt
for local rings with respect to its maximal ideal.
Main results #
PowerSeries.exists_isWeierstrassDivision
: Weierstrass division ([Was97], Proposition 7.2): letf
,g
be power series over a complete local ring, such that the image ofg
in the residue field is not zero. Letn
be the order of the image ofg
in the residue field. Then there exists a power seriesq
and a polynomialr
of degree< n
, such thatf = g * q + r
.PowerSeries.IsWeierstrassDivision.elim
,PowerSeries.IsWeierstrassDivision.unique
:q
andr
in the Weierstrass division are unique.PowerSeries.exists_isWeierstrassFactorization
: Weierstrass preparation theorem ([Was97], Theorem 7.3): letg
be a power series over a complete local ring, such that the image ofg
in the residue field is not zero. Then there exists a distinguished polynomialf
and a power seriesh
which is a unit, such thatg = f * h
.PowerSeries.IsWeierstrassFactorization.elim
,PowerSeries.IsWeierstrassFactorization.unique
:f
andh
in Weierstrass preparation theorem are unique.
References #
Weierstrass division #
Let f
, g
be power series over A
, I
be an ideal of A
,
PowerSeries.IsWeierstrassDivisionAt f g q r I
is a Prop
which asserts that a power series
q
and a polynomial r
of degree < n
satisfy f = g * q + r
, where n
is the order of the
image of g
in (A / I)⟦X⟧
(defined to be zero if such image is zero, in which case
it's mathematically not considered).
Instances For
Version of PowerSeries.IsWeierstrassDivisionAt
for local rings with respect to
its maximal ideal.
Equations
- f.IsWeierstrassDivision g q r = f.IsWeierstrassDivisionAt g q r (IsLocalRing.maximalIdeal A)
Instances For
PowerSeries.IsWeierstrassDivisorAt g I
is a Prop
which asserts that the n
-th coefficient
of g
is a unit, where n
is the order of the
image of g
in (A / I)⟦X⟧
(defined to be zero if such image is zero, in which case
it's mathematically not considered).
This property guarantees that if the ring is I
-adic complete, then g
can be used as a divisor
in Weierstrass division (PowerSeries.IsWeierstrassDivisorAt.isWeierstrassDivisionAt_div_mod
).
Equations
- g.IsWeierstrassDivisorAt I = IsUnit ((PowerSeries.coeff A ((PowerSeries.map (Ideal.Quotient.mk I)) g).order.toNat) g)
Instances For
Version of PowerSeries.IsWeierstrassDivisorAt
for local rings with respect to
its maximal ideal.
Equations
Instances For
If g
is a power series over a local ring such that
its image in the residue field is not zero, then g
can be used as a Weierstrass divisor.
The inductively constructed sequence qₖ
in the proof of Weierstrass division.
Equations
Instances For
The (bundled version of) coefficient of the limit q
of the
inductively constructed sequence qₖ
in the proof of Weierstrass division.
Equations
Instances For
The limit q
of the
inductively constructed sequence qₖ
in the proof of Weierstrass division.
Equations
- H.div f = PowerSeries.mk fun (i : ℕ) => ↑(H.divCoeff f i)
Instances For
The remainder r
in the proof of Weierstrass division.
Equations
- H.mod f = PowerSeries.trunc ((PowerSeries.map (Ideal.Quotient.mk I)) g).order.toNat (f - g * H.div f)
Instances For
If the ring is I
-adic complete, then g
can be used as a divisor in Weierstrass division.
If g * q = r
for some power series q
and some polynomial r
whose degree is < n
,
then q
and r
are all zero. This implies the uniqueness of Weierstrass division.
If g * q + r = g * q' + r'
for some power series q
, q'
and some polynomials r
, r'
whose degrees are < n
, then q = q'
and r = r'
are all zero.
This implies the uniqueness of Weierstrass division.
Weierstrass division ([Was97], Proposition 7.2): let f
, g
be
power series over a complete local ring, such that
the image of g
in the residue field is not zero. Let n
be the order of the image of g
in the
residue field. Then there exists a power series q
and a polynomial r
of degree < n
, such that
f = g * q + r
.
The quotient q
in Weierstrass division, denoted by f /ʷ g
. Note that when the image of
g
in the residue field is zero, this is defined to be zero.
Equations
- f /ʷ g = if hg : (PowerSeries.map (IsLocalRing.residue A)) g ≠ 0 then PowerSeries.IsWeierstrassDivisorAt.div ⋯ f else 0
Instances For
The remainder r
in Weierstrass division, denoted by f %ʷ g
. Note that when the image of
g
in the residue field is zero, this is defined to be zero.
Equations
- f %ʷ g = if hg : (PowerSeries.map (IsLocalRing.residue A)) g ≠ 0 then PowerSeries.IsWeierstrassDivisorAt.mod ⋯ f else 0
Instances For
The quotient q
in Weierstrass division, denoted by f /ʷ g
. Note that when the image of
g
in the residue field is zero, this is defined to be zero.
Equations
- PowerSeries.«term_/ʷ_» = Lean.ParserDescr.trailingNode `PowerSeries.«term_/ʷ_» 70 70 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " /ʷ ") (Lean.ParserDescr.cat `term 71))
Instances For
The remainder r
in Weierstrass division, denoted by f %ʷ g
. Note that when the image of
g
in the residue field is zero, this is defined to be zero.
Equations
- PowerSeries.«term_%ʷ_» = Lean.ParserDescr.trailingNode `PowerSeries.«term_%ʷ_» 70 70 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " %ʷ ") (Lean.ParserDescr.cat `term 71))
Instances For
The quotient q
and the remainder r
in the Weierstrass division are unique.
This result is stated using two PowerSeries.IsWeierstrassDivision
assertions, and only requires
the ring being Hausdorff with respect to the maximal ideal. If you want q
and r
equal to
f /ʷ g
and f %ʷ g
, use PowerSeries.IsWeierstrassDivision.unique
instead, which requires the ring being complete with respect to the maximal ideal.
If q
and r
are quotient and remainder in the Weierstrass division 0 / g
, then they are
equal to 0
.
If q
and r
are quotient and remainder in the Weierstrass division f / g
, then they are
equal to f /ʷ g
and f %ʷ g
.
Weierstrass preparation theorem #
If f
is a polynomial over A
, g
and h
are power series over A
,
then PowerSeries.IsWeierstrassFactorizationAt g f h I
is a Prop
which asserts that f
is
distingushed at I
, h
is a unit, such that g = f * h
.
- isDistinguishedAt : f.IsDistinguishedAt I
- isUnit : IsUnit h
Instances For
Version of PowerSeries.IsWeierstrassFactorizationAt
for local rings with respect to
its maximal ideal.
Equations
Instances For
Weierstrass preparation theorem ([Was97], Theorem 7.3):
let g
be a power series over a complete local ring,
such that the image of g
in the residue field is not zero. Then there exists a distinguished
polynomial f
and a power series h
which is a unit, such that g = f * h
.
The f
in the Weierstrass preparation theorem.
Equations
Instances For
The h
in the Weierstrass preparation theorem.
Equations
Instances For
The f
and h
in the Weierstrass preparation theorem are unique.
This result is stated using two PowerSeries.IsWeierstrassFactorization
assertions, and only
requires the ring being Hausdorff with respect to the maximal ideal. If you want f
and h
equal
to PowerSeries.weierstrassDistinguished
and PowerSeries.weierstrassUnit
,
use PowerSeries.IsWeierstrassFactorization.unique
instead, which requires the ring being
complete with respect to the maximal ideal.
The f
and h
in Weierstrass preparation theorem are equal
to PowerSeries.weierstrassDistinguished
and PowerSeries.weierstrassUnit
.