Substitutions in power series #
A (possibly multivariate) power series can be substituted into a (univariate) power series if and only if its constant coefficient is nilpotent.
This is a particularization of the substitution of multivariate power series to the case of univariate power series.
Because of the special API for PowerSeries
, some results for MvPowerSeries
do not immediately apply and a “primed” version is provided here.
(Possibly multivariate) power series which can be substituted in a PowerSeries
.
Equations
- PowerSeries.HasSubst a = IsNilpotent ((MvPowerSeries.constantCoeff τ S) a)
Instances For
A variant of HasSubst.of_constantCoeff_zero
for PowerSeries
to avoid the expansion of Unit
.
The univariate X : R⟦X⟧
can be substituted in power series
This lemma is added because simp
doesn't find it from HasSubst.X
.
A variant of HasSubst.monomial
to avoid the expansion of Unit
.
A variant of HasSubst.zero
to avoid the expansion of Unit
.
Families of PowerSeries
that can be substituted, as an Ideal
.
Equations
- PowerSeries.HasSubst.ideal = { carrier := setOf PowerSeries.HasSubst, add_mem' := ⋯, zero_mem' := ⋯, smul_mem' := ⋯ }
Instances For
A more general version of HasSubst.smul
.
Substitution of power series into a power series.
Equations
- PowerSeries.subst a f = MvPowerSeries.subst (fun (x : Unit) => a) f
Instances For
Substitution of power series into a power series, as an AlgHom
.
Equations
Instances For
Rewrite PowerSeries.substAlgHom
as PowerSeries.aeval
.
Its use is discouraged because it introduces a topology and might lead into awkward comparisons.