Linear topology on the ring of multivariate power series #
MvPowerSeries.LinearTopology.basis
: the ideals of the ring of multivariate power series all coefficients the exponent of which is smaller than some bound vanish.MvPowerSeries.LinearTopology.hasBasis_nhds_zero
: the two-sided ideals fromMvPowerSeries.LinearTopology.basis
form a basis of neighborhoods of0
if the topology ofR
is (left and right) linear.
Instances : #
If R
has a linear topology, then the product topology on MvPowerSeries σ R
is a linear topology.
This applies in particular when R
has the discrete topology.
Note #
If we had an analogue of PolynomialModule
for power series,
meaning that we could consider the R⟦X⟧
-module M⟦X⟧
when M
is an R
-module,
then one could prove that M⟦X⟧
is linearly topologized over R⟦X⟧
whenever M
is linearly topologized over R
.
To recover the ring case, it would remain to show that the isomorphism between
Rᵐᵒᵖ⟦X⟧
and R⟦X⟧ᵐᵒᵖ
identifies their respective actions on R⟦X⟧
.
(And likewise in the multivariate case.)
The underlying family for the basis of ideals in a multivariate power series ring.
Equations
- MvPowerSeries.LinearTopology.basis σ R Jd = TwoSidedIdeal.mk' {f : MvPowerSeries σ R | ∀ e ≤ Jd.2, (MvPowerSeries.coeff R e) f ∈ Jd.1} ⋯ ⋯ ⋯ ⋯ ⋯
Instances For
A power series f
belongs to the twosided ideal basis σ R ⟨J, d⟩
if and only if coeff R e f ∈ J
for all e ≤ d
.
If the ring R
is endowed with a linear topology, then the sets ↑basis σ R (J, d)
,
for J : TwoSidedIdeal R
which are neighborhoods of 0 : R
and d : σ →₀ ℕ
,
constitute a basis of neighborhoods of 0 : MvPowerSeries σ R
for the product topology.
The topology on MvPowerSeries
is a left linear topology
when the ring of coefficients has a linar topology.
The topology on MvPowerSeries
is a right linear topology
when the ring of coefficients has a linear topology.