Documentation

Mathlib.RingTheory.MvPowerSeries.Trunc

Formal (multivariate) power series - Truncation #

MvPowerSeries.trunc n φ truncates a formal multivariate power series to the multivariate polynomial that has the same coefficients as φ, for all m < n, and 0 otherwise.

Note that here, m and n have types σ →₀ ℕ, so that m < n means that m ≠ n and m s ≤ n s for all s : σ.

def MvPowerSeries.truncFun {σ : Type u_1} {R : Type u_2} [CommSemiring R] (n : σ →₀ ) (φ : MvPowerSeries σ R) :

Auxiliary definition for the truncation function.

Equations
Instances For
    theorem MvPowerSeries.coeff_truncFun {σ : Type u_1} {R : Type u_2} [CommSemiring R] (n : σ →₀ ) (m : σ →₀ ) (φ : MvPowerSeries σ R) :
    MvPolynomial.coeff m (MvPowerSeries.truncFun n φ) = if m < n then (MvPowerSeries.coeff R m) φ else 0
    def MvPowerSeries.trunc {σ : Type u_1} (R : Type u_2) [CommSemiring R] (n : σ →₀ ) :

    The nth truncation of a multivariate formal power series to a multivariate polynomial

    Equations
    Instances For
      theorem MvPowerSeries.coeff_trunc {σ : Type u_1} {R : Type u_2} [CommSemiring R] (n : σ →₀ ) (m : σ →₀ ) (φ : MvPowerSeries σ R) :
      MvPolynomial.coeff m ((MvPowerSeries.trunc R n) φ) = if m < n then (MvPowerSeries.coeff R m) φ else 0
      @[simp]
      theorem MvPowerSeries.trunc_one {σ : Type u_1} {R : Type u_2} [CommSemiring R] (n : σ →₀ ) (hnn : n 0) :
      @[simp]
      theorem MvPowerSeries.trunc_c {σ : Type u_1} {R : Type u_2} [CommSemiring R] (n : σ →₀ ) (hnn : n 0) (a : R) :
      (MvPowerSeries.trunc R n) ((MvPowerSeries.C σ R) a) = MvPolynomial.C a