Documentation

Mathlib.RingTheory.PowerSeries.Exp

Exponential Power Series #

This file defines the exponential power series exp A = ∑ Xⁿ/n! over ℚ-algebras and develops its key properties, including the fundamental differential equation (exp A)' = exp A, a uniqueness characterization, and the functional equation for multiplication.

Main definitions #

Main results #

def PowerSeries.exp (A : Type u_1) [Ring A] [Algebra A] :

Power series for the exponential function at zero.

Equations
Instances For
    @[simp]
    theorem PowerSeries.coeff_exp {A : Type u_1} [Ring A] [Algebra A] (n : ) :
    (coeff n) (exp A) = (algebraMap A) (1 / n.factorial)
    @[simp]
    @[simp]
    theorem PowerSeries.map_exp {A : Type u_1} {A' : Type u_2} [Ring A] [Ring A'] [Algebra A] [Algebra A'] (f : A →+* A') :
    (map f) (exp A) = exp A'

    Derivative of exp #

    Uniqueness characterization #

    A power series with derivative equal to itself and constant term 1 must be exp.

    The proof uses induction on coefficients: if f' = f and f(0) = 1, then coeff (n+1) f * (n+1) = coeff n f, which determines all coefficients uniquely.

    Order and invertibility #

    theorem PowerSeries.isUnit_exp (A : Type u_4) [Ring A] [Algebra A] :
    @[simp]
    theorem PowerSeries.order_exp (A : Type u_4) [Ring A] [Algebra A] [Nontrivial A] :
    (exp A).order = 0
    theorem PowerSeries.exp_mul_exp_eq_exp_add {A : Type u_4} [CommRing A] [Algebra A] (a b : A) :
    (rescale a) (exp A) * (rescale b) (exp A) = (rescale (a + b)) (exp A)

    Shows that $e^{aX} * e^{bX} = e^{(a + b)X}$

    Shows that $e^{x} * e^{-x} = 1$

    theorem PowerSeries.exp_pow_eq_rescale_exp {A : Type u_4} [CommRing A] [Algebra A] (k : ) :
    exp A ^ k = (rescale k) (exp A)

    Shows that $(e^{X})^k = e^{kX}$.

    theorem PowerSeries.exp_pow_sum {A : Type u_4} [CommRing A] [Algebra A] (n : ) :
    kFinset.range n, exp A ^ k = mk fun (p : ) => kFinset.range n, k ^ p * (algebraMap A) (↑p.factorial)⁻¹

    Shows that $\sum_{k = 0}^{n - 1} (e^{X})^k = \sum_{p = 0}^{\infty} \sum_{k = 0}^{n - 1} \frac{k^p}{p!}X^p$.