mathlib3 documentation

ring_theory.polynomial.hermite.gaussian

Hermite polynomials and Gaussians #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file shows that the Hermite polynomial hermite n is (up to sign) the polynomial factor occurring in the nth derivative of a gaussian.

Results #

References #

theorem polynomial.deriv_gaussian_eq_hermite_mul_gaussian (n : ) (x : ) :
deriv^[n] (λ (y : ), rexp (-(y ^ 2 / 2))) x = (-1) ^ n * (polynomial.aeval x) (polynomial.hermite n) * rexp (-(x ^ 2 / 2))

hermite n is (up to sign) the factor appearing in deriv^[n] of a gaussian

theorem polynomial.hermite_eq_deriv_gaussian (n : ) (x : ) :
(polynomial.aeval x) (polynomial.hermite n) = (-1) ^ n * deriv^[n] (λ (y : ), rexp (-(y ^ 2 / 2))) x / rexp (-(x ^ 2 / 2))
theorem polynomial.hermite_eq_deriv_gaussian' (n : ) (x : ) :
(polynomial.aeval x) (polynomial.hermite n) = (-1) ^ n * deriv^[n] (λ (y : ), rexp (-(y ^ 2 / 2))) x * rexp (x ^ 2 / 2)