Documentation

Mathlib.RingTheory.HahnSeries.HEval

Evaluation of power series in Hahn Series #

We describe a class of ring homomorphisms from formal power series to Hahn series, given by substitution of the generating variable to an element of strictly positive order.

Main Definitions #

TODO #

@[reducible, inline]

A summable family given by scalar multiples of powers of a positive order Hahn series.

The scalar multiples are given by the coefficients of a power series.

Equations
Instances For

    The R-algebra homomorphism from R[[X]] to HahnSeries Γ R given by sending the power series variable X to a positive order element x and extending to infinite sums.

    Equations
    Instances For
      theorem PowerSeries.heval_mul {Γ : Type u_1} {R : Type u_3} [AddCommMonoid Γ] [LinearOrder Γ] [IsOrderedCancelAddMonoid Γ] [CommRing R] (x : HahnSeries Γ R) {a b : PowerSeries R} :
      (heval x) (a * b) = (heval x) a * (heval x) b
      theorem PowerSeries.heval_C {Γ : Type u_1} {R : Type u_3} [AddCommMonoid Γ] [LinearOrder Γ] [IsOrderedCancelAddMonoid Γ] [CommRing R] (x : HahnSeries Γ R) (r : R) :
      (heval x) (C r) = r 1
      theorem PowerSeries.heval_X {Γ : Type u_1} {R : Type u_3} [AddCommMonoid Γ] [LinearOrder Γ] [IsOrderedCancelAddMonoid Γ] [CommRing R] (x : HahnSeries Γ R) (hx : 0 < x.orderTop) :
      (heval x) X = x
      theorem PowerSeries.heval_unit {Γ : Type u_1} {R : Type u_3} [AddCommMonoid Γ] [LinearOrder Γ] [IsOrderedCancelAddMonoid Γ] [CommRing R] (x : HahnSeries Γ R) (u : (PowerSeries R)ˣ) :
      IsUnit ((heval x) u)