Documentation

Mathlib.RingTheory.MvPowerSeries.PiTopology

Product topology on multivariate power series #

Let R be with Semiring R and TopologicalSpace R In this file we define the topology on MvPowerSeries σ R that corresponds to the simple convergence on its coefficients. It is the coarsest topology for which all coefficient maps are continuous.

When R has UniformSpace R, we define the corresponding uniform structure.

This topology can be included by writing open scoped MvPowerSeries.WithPiTopology.

When the type of coefficients has the discrete topology, it corresponds to the topology defined by [Bou90], chapter 4, §4, n°2.

It is not the adic topology in general.

Main results #

TODO: add the similar result for the series of homogeneous components.

Instances #

theorem MvPowerSeries.WithPiTopology.tendsto_iff_coeff_tendsto {σ : Type u_1} {R : Type u_2} [TopologicalSpace R] [Semiring R] {ι : Type u_3} (f : ιMvPowerSeries σ R) (u : Filter ι) (g : MvPowerSeries σ R) :
Filter.Tendsto f u (nhds g) ∀ (d : σ →₀ ), Filter.Tendsto (fun (i : ι) => (MvPowerSeries.coeff R d) (f i)) u (nhds ((MvPowerSeries.coeff R d) g))

A family of power series converges iff it converges coefficientwise

The semiring topology on MvPowerSeries of a topological semiring

The ring topology on MvPowerSeries of a topological ring

theorem MvPowerSeries.WithPiTopology.variables_tendsto_zero {σ : Type u_1} {R : Type u_2} [TopologicalSpace R] [Semiring R] :
Filter.Tendsto (fun (x : σ) => MvPowerSeries.X x) Filter.cofinite (nhds 0)

The powers of a MvPowerSeries converge to 0 iff its constant coefficient is nilpotent. N. Bourbaki, Algebra II, [Bou90] (chap. 4, §4, n°2, corollaire de la prop. 3)

A multivariate power series is the sum (in the sense of summable families) of its monomials

theorem MvPowerSeries.WithPiTopology.as_tsum {σ : Type u_1} {R : Type u_2} [TopologicalSpace R] [Semiring R] [T2Space R] (f : MvPowerSeries σ R) :
f = ∑' (d : σ →₀ ), (MvPowerSeries.monomial R d) ((MvPowerSeries.coeff R d) f)

If the coefficient space is T2, then the multivariate power series is tsum of its monomials

The componentwise uniformity on MvPowerSeries

Equations
Instances For

    Coefficients of a multivariate power series are uniformly continuous

    Completeness of the uniform structure on MvPowerSeries