Documentation

Mathlib.RingTheory.Polynomial.Hermite.Basic

Hermite polynomials #

This file defines Polynomial.hermite n, the nth probabilists' Hermite polynomial.

Main definitions #

Results #

References #

The recursion hermite (n+1) = (x - d/dx) (hermite n)

Lemmas about Polynomial.coeff #

theorem Polynomial.coeff_hermite_of_lt {n k : Nat} (hnk : LT.lt n k) :
Eq ((hermite n).coeff k) 0
theorem Polynomial.coeff_hermite_of_odd_add {n k : Nat} (hnk : Odd (HAdd.hAdd n k)) :
Eq ((hermite n).coeff k) 0
@[irreducible]

Because of coeff_hermite_of_odd_add, every nonzero coefficient is described as follows.