Gaussian integral #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We prove various versions of the formula for the Gaussian integral:
integral_gaussian
: for realb
we have∫ x:ℝ, exp (-b * x^2) = sqrt (π / b)
.integral_gaussian_complex
: for complexb
with0 < re b
we have∫ x:ℝ, exp (-b * x^2) = (π / b) ^ (1 / 2)
.integral_gaussian_Ioi
andintegral_gaussian_complex_Ioi
: variants for integrals overIoi 0
.complex.Gamma_one_half_eq
: the formulaΓ (1 / 2) = √π
.
We also prove, more generally, that the Fourier transform of the Gaussian is another Gaussian:
integral_cexp_neg_mul_sq_add_const
: for all complexb
andc
with0 < re b
we have∫ (x : ℝ), exp (-b * (x + c) ^ 2) = (π / b) ^ (1 / 2)
.fourier_transform_gaussian
: for all complexb
andt
with0 < re b
, we have∫ x:ℝ, exp (I * t * x) * exp (-b * x^2) = (π / b) ^ (1 / 2) * exp (-t ^ 2 / (4 * b))
.fourier_transform_gaussian_pi
: a variant withb
andt
scaled to give a more symmetric statement, and formulated in terms of the Fourier transform operator𝓕
.
As an application, in real.tsum_exp_neg_mul_int_sq
and complex.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
number_theory.modular_forms.jacobi_theta
.)
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)
.