Hermite polynomials #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines polynomial.hermite n
, the nth probabilist's Hermite polynomial.
Main definitions #
polynomial.hermite n
: then
th probabilist's 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 nth probabilist's Hermite polynomial
Equations
@[simp]
The recursion hermite (n+1) = (x - d/dx) (hermite n)
theorem
polynomial.hermite_eq_iterate
(n : ℕ) :
polynomial.hermite n = (λ (p : polynomial ℤ), polynomial.X * p - ⇑polynomial.derivative p)^[n] 1
Lemmas about polynomial.coeff
#
theorem
polynomial.coeff_hermite_succ_zero
(n : ℕ) :
(polynomial.hermite (n + 1)).coeff 0 = -(polynomial.hermite n).coeff 1
theorem
polynomial.coeff_hermite_succ_succ
(n k : ℕ) :
(polynomial.hermite (n + 1)).coeff (k + 1) = (polynomial.hermite n).coeff k - (↑k + 2) * (polynomial.hermite n).coeff (k + 2)
@[simp]
@[simp]
theorem
polynomial.coeff_hermite_of_odd_add
{n k : ℕ}
(hnk : odd (n + k)) :
(polynomial.hermite n).coeff k = 0