Documentation

Mathlib.Analysis.SpecialFunctions.Gaussian

Gaussian integral #

We prove various versions of the formula for the Gaussian integral:

We also prove, more generally, that the Fourier transform of the Gaussian is another Gaussian:

As an application, in Real.tsum_exp_neg_mul_int_sq and cCmplex.tsum_exp_neg_mul_int_sq, we use Poisson summation to prove the identity ∑' (n : ℤ), exp (-π * a * n ^ 2) = 1 / a ^ (1 / 2) * ∑' (n : ℤ), exp (-π / a * n ^ 2) for positive real a, or complex a with positive real part. (See also NumberTheory.ModularForms.JacobiTheta.)

theorem exp_neg_mul_sq_isLittleO_exp_neg {b : } (hb : 0 < b) :
(fun x => Real.exp (-b * x ^ 2)) =o[Filter.atTop] fun x => Real.exp (-x)
theorem rpow_mul_exp_neg_mul_sq_isLittleO_exp_neg {b : } (hb : 0 < b) (s : ) :
(fun x => x ^ s * Real.exp (-b * x ^ 2)) =o[Filter.atTop] fun x => Real.exp (-(1 / 2) * x)
theorem integrableOn_rpow_mul_exp_neg_mul_sq {b : } (hb : 0 < b) {s : } (hs : -1 < s) :
MeasureTheory.IntegrableOn (fun x => x ^ s * Real.exp (-b * x ^ 2)) (Set.Ioi 0)
theorem integrable_rpow_mul_exp_neg_mul_sq {b : } (hb : 0 < b) {s : } (hs : -1 < s) :
MeasureTheory.Integrable fun x => x ^ s * Real.exp (-b * x ^ 2)
theorem integrable_exp_neg_mul_sq {b : } (hb : 0 < b) :
theorem integrable_mul_exp_neg_mul_sq {b : } (hb : 0 < b) :
theorem norm_cexp_neg_mul_sq (b : ) (x : ) :
Complex.exp (-b * x ^ 2) = Real.exp (-b.re * x ^ 2)
theorem integrable_cexp_neg_mul_sq {b : } (hb : 0 < b.re) :
theorem integrable_mul_cexp_neg_mul_sq {b : } (hb : 0 < b.re) :
MeasureTheory.Integrable fun x => x * Complex.exp (-b * x ^ 2)
theorem integral_mul_cexp_neg_mul_sq {b : } (hb : 0 < b.re) :
∫ (r : ) in Set.Ioi 0, r * Complex.exp (-b * r ^ 2) = (2 * b)⁻¹
theorem integral_gaussian_sq_complex {b : } (hb : 0 < b.re) :
(∫ (x : ), Complex.exp (-b * x ^ 2)) ^ 2 = Real.pi / b

The square of the Gaussian integral ∫ x:ℝ, exp (-b * x^2) is equal to π / b.

theorem integral_gaussian (b : ) :
∫ (x : ), Real.exp (-b * x ^ 2) = Real.sqrt (Real.pi / b)
theorem continuousAt_gaussian_integral (b : ) (hb : 0 < b.re) :
ContinuousAt (fun c => ∫ (x : ), Complex.exp (-c * x ^ 2)) b
theorem integral_gaussian_complex {b : } (hb : 0 < b.re) :
∫ (x : ), Complex.exp (-b * x ^ 2) = (Real.pi / b) ^ (1 / 2)
theorem integral_gaussian_complex_Ioi {b : } (hb : 0 < b.re) :
∫ (x : ) in Set.Ioi 0, Complex.exp (-b * x ^ 2) = (Real.pi / b) ^ (1 / 2) / 2
theorem integral_gaussian_Ioi (b : ) :
∫ (x : ) in Set.Ioi 0, Real.exp (-b * x ^ 2) = Real.sqrt (Real.pi / b) / 2

The special-value formula Γ(1/2) = √π, which is equivalent to the Gaussian integral.

The special-value formula Γ(1/2) = √π, which is equivalent to the Gaussian integral.

Fourier transform of the Gaussian integral #

The integral of the Gaussian function over the vertical edges of a rectangle with vertices at (±T, 0) and (±T, c).

Instances For
    theorem GaussianFourier.norm_cexp_neg_mul_sq_add_mul_I (b : ) (c : ) (T : ) :
    Complex.exp (-b * (T + c * Complex.I) ^ 2) = Real.exp (-(b.re * T ^ 2 - 2 * b.im * c * T - b.re * c ^ 2))

    Explicit formula for the norm of the Gaussian function along the vertical edges.

    theorem GaussianFourier.norm_cexp_neg_mul_sq_add_mul_I' {b : } (hb : b.re 0) (c : ) (T : ) :
    Complex.exp (-b * (T + c * Complex.I) ^ 2) = Real.exp (-(b.re * (T - b.im * c / b.re) ^ 2 - c ^ 2 * (b.im ^ 2 / b.re + b.re)))
    theorem GaussianFourier.verticalIntegral_norm_le {b : } (hb : 0 < b.re) (c : ) {T : } (hT : 0 T) :
    GaussianFourier.verticalIntegral b c T 2 * |c| * Real.exp (-(b.re * T ^ 2 - 2 * |b.im| * |c| * T - b.re * c ^ 2))
    theorem GaussianFourier.integral_cexp_neg_mul_sq_add_real_mul_I {b : } (hb : 0 < b.re) (c : ) :
    ∫ (x : ), Complex.exp (-b * (x + c * Complex.I) ^ 2) = (Real.pi / b) ^ (1 / 2)
    theorem integral_cexp_neg_mul_sq_add_const {b : } (hb : 0 < b.re) (c : ) :
    ∫ (x : ), Complex.exp (-b * (x + c) ^ 2) = (Real.pi / b) ^ (1 / 2)
    theorem fourier_transform_gaussian {b : } (hb : 0 < b.re) (t : ) :
    ∫ (x : ), Complex.exp (Complex.I * t * x) * Complex.exp (-b * x ^ 2) = Complex.exp (-t ^ 2 / (4 * b)) * (Real.pi / b) ^ (1 / 2)
    theorem fourier_transform_gaussian_pi {b : } (hb : 0 < b.re) :
    (Real.fourierIntegral fun x => Complex.exp (-Real.pi * b * x ^ 2)) = fun t => 1 / b ^ (1 / 2) * Complex.exp (-Real.pi / b * t ^ 2)

    Poisson summation applied to the Gaussian #

    theorem tendsto_rpow_abs_mul_exp_neg_mul_sq_cocompact {a : } (ha : 0 < a) (s : ) :
    Filter.Tendsto (fun x => |x| ^ s * Real.exp (-a * x ^ 2)) (Filter.cocompact ) (nhds 0)
    theorem isLittleO_exp_neg_mul_sq_cocompact {a : } (ha : 0 < a.re) (s : ) :
    (fun x => Complex.exp (-a * x ^ 2)) =o[Filter.cocompact ] fun x => |x| ^ s
    theorem Complex.tsum_exp_neg_mul_int_sq {a : } (ha : 0 < a.re) :
    ∑' (n : ), Complex.exp (-Real.pi * a * n ^ 2) = 1 / a ^ (1 / 2) * ∑' (n : ), Complex.exp (-Real.pi / a * n ^ 2)
    theorem Real.tsum_exp_neg_mul_int_sq {a : } (ha : 0 < a) :
    ∑' (n : ), Real.exp (-Real.pi * a * n ^ 2) = 1 / a ^ (1 / 2) * ∑' (n : ), Real.exp (-Real.pi / a * n ^ 2)