Hermite polynomials #
This file defines Polynomial.hermite n
, the n
th probabilists' Hermite polynomial.
Main definitions #
Polynomial.hermite n
: then
th probabilists' Hermite polynomial, defined recursively as aPolynomial ℤ
Results #
Polynomial.hermite_succ
: the recursionhermite (n+1) = (x - d/dx) (hermite n)
Polynomial.coeff_hermite_explicit
: a closed formula for (nonvanishing) coefficients in terms of binomial coefficients and double factorials.Polynomial.coeff_hermite_of_odd_add
: forn
,k
wheren+k
is odd,(hermite n).coeff k
is zero.Polynomial.coeff_hermite_of_even_add
: a closed formula for(hermite n).coeff k
whenn+k
is even, equivalent toPolynomial.coeff_hermite_explicit
.Polynomial.monic_hermite
: for alln
,hermite n
is monic.Polynomial.degree_hermite
: for alln
,hermite n
has degreen
.
References #
the probabilists' Hermite polynomials.
Equations
Instances For
theorem
Polynomial.hermite_succ
(n : Nat)
:
Eq (hermite (HAdd.hAdd n 1)) (HSub.hSub (HMul.hMul X (hermite n)) (DFunLike.coe derivative (hermite n)))
The recursion hermite (n+1) = (x - d/dx) (hermite n)
theorem
Polynomial.hermite_eq_iterate
(n : Nat)
:
Eq (hermite n) (Nat.iterate (fun (p : Polynomial Int) => HSub.hSub (HMul.hMul X p) (DFunLike.coe derivative p)) n 1)
Lemmas about Polynomial.coeff
#
@[irreducible]
Because of coeff_hermite_of_odd_add
, every nonzero coefficient is described as follows.