The Fourier transform #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We set up the Fourier transform for complex-valued functions on finite-dimensional spaces.
Design choices #
In namespace vector_fourier, we define the Fourier integral in the following context:
𝕜is a commutative ring.VandWare𝕜-modules.eis a unitary additive character of𝕜, i.e. a homomorphism(multiplicative 𝕜) →* circle.μis a measure onV.Lis a𝕜-bilinear formV × W → 𝕜.Eis a complete normedℂ-vector space.
With these definitions, we define fourier_integral to be the map from functions V → E to
functions W → E that sends f to
λ w, ∫ v in V, e [-L v w] • f v ∂μ,
where e [x] is notational sugar for (e (multiplicative.of_add x) : ℂ) (available in locale
fourier_transform). This includes the cases W is the dual of V and L is the canonical
pairing, or W = V and L is a bilinear form (e.g. an inner product).
In namespace fourier, we consider the more familiar special case when V = W = 𝕜 and L is the
multiplication map (but still allowing 𝕜 to be an arbitrary ring equipped with a measure).
The most familiar case of all is when V = W = 𝕜 = ℝ, L is multiplication, μ is volume, and
e is real.fourier_char, i.e. the character λ x, exp ((2 * π * x) * I). The Fourier integral
in this case is defined as real.fourier_integral.
Main results #
At present the only nontrivial lemma we prove is continuous_fourier_integral, stating that the
Fourier transform of an integrable function is continuous (under mild assumptions).
Fourier theory for functions on general vector spaces #
The Fourier transform integral for f : V → E, with respect to a bilinear form L : V × W → 𝕜
and an additive character e.
The uniform norm of the Fourier integral of f is bounded by the L¹ norm of f.
The Fourier integral converts right-translation into scalar multiplication by a phase factor.
For any w, the Fourier integral is convergent iff f is integrable.
The Fourier integral of an L^1 function is a continuous function.
Fourier theory for functions on 𝕜 #
The Fourier transform integral for f : 𝕜 → E, with respect to the measure μ and additive
character e.
Equations
- fourier.fourier_integral e μ f w = vector_fourier.fourier_integral e μ (linear_map.mul 𝕜 𝕜) f w
The uniform norm of the Fourier transform of f is bounded by the L¹ norm of f.
The Fourier transform converts right-translation into scalar multiplication by a phase factor.
The standard additive character of ℝ, given by λ x, exp (2 * π * x * I).
Equations
- real.fourier_char = {to_fun := λ (z : multiplicative ℝ), ⇑exp_map_circle (2 * real.pi * ⇑multiplicative.to_add z), map_one' := real.fourier_char._proof_1, map_mul' := real.fourier_char._proof_2}
The Fourier integral for f : ℝ → E, with respect to the standard additive character and
measure on ℝ.