Documentation

Mathlib.RingTheory.PowerSeries.PiTopology

Product topology on power series #

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

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

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

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

It corresponds with the adic topology but this is not proved here.

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

Instances #

Coefficients are continuous

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

A family of power series converges iff it converges coefficientwise

The product uniformity on PowerSeries

Equations
Instances For

    Coefficients are uniformly continuous

    Completeness of the uniform structure on PowerSeries

    The powers of a PowerSeries 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 power series is the sum (in the sense of summable families) of its monomials

    theorem PowerSeries.as_tsum {R : Type u_1} [Semiring R] [TopologicalSpace R] [T2Space R] (f : PowerSeries R) :
    f = ∑' (d : ), (PowerSeries.monomial R d) ((PowerSeries.coeff R d) f)

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