Fourier analysis on the additive circle #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains basic results on Fourier series for functions on the additive circle
add_circle T = ℝ / ℤ • T
.
Main definitions #
haar_add_circle
, Haar measure onadd_circle T
, normalized to have total measure1
. (Note that this is not the same normalisation as the standard measure defined inintegral.periodic
, so we do not declare it as ameasure_space
instance, to avoid confusion.)- for
n : ℤ
,fourier n
is the monomialλ x, exp (2 π i n x / T)
, bundled as a continuous map fromadd_circle T
toℂ
. fourier_basis
is the Hilbert basis ofLp ℂ 2 haar_add_circle
given by the images of the monomialsfourier n
.fourier_coeff f n
, forf : add_circle T → E
(withE
a complete normedℂ
-vector space), is then
-th Fourier coefficient off
, defined as an integral overadd_circle T
. The lemmafourier_coeff_eq_interval_integral
expresses this as an integral over[a, a + T]
for any reala
.fourier_coeff_on
, forf : ℝ → E
anda < b
reals, is then
-th Fourier coefficient of the unique periodic function of periodb - a
which agrees withf
on(a, b]
. The lemmafourier_coeff_on_eq_integral
expresses this as an integral over[a, b]
.
Main statements #
The theorem span_fourier_closure_eq_top
states that the span of the monomials fourier n
is
dense in C(add_circle T, ℂ)
, i.e. that its submodule.topological_closure
is ⊤
. This follows
from the Stone-Weierstrass theorem after checking that the span is a subalgebra, is closed under
conjugation, and separates points.
Using this and general theory on approximation of Lᵖ functions by continuous functions, we deduce
(span_fourier_Lp_closure_eq_top
) that for any 1 ≤ p < ∞
, the span of the Fourier monomials is
dense in the Lᵖ space of add_circle T
. For p = 2
we show (orthonormal_fourier
) that the
monomials are also orthonormal, so they form a Hilbert basis for L², which is named as
fourier_basis
; in particular, for L²
functions f
, the Fourier series of f
converges to f
in the L²
topology (has_sum_fourier_series_L2
). Parseval's identity, tsum_sq_fourier_coeff
, is
a direct consequence.
For continuous maps f : add_circle T → ℂ
, the theorem
continuous_map.has_sum_fourier_series_of_summable
states that if the sequence of Fourier
coefficients of f
is summable, then the Fourier series ∑ (i:ℤ), f.fourier_coeff i * fourier i
converges to f
in the uniform-convergence topology of C(add_circle T, ℂ)
.
Map from add_circle
to circle
#
The canonical map λ x, exp (2 π i x / T)
from ℝ / ℤ • T
to the unit circle in ℂ
.
If T = 0
we understand this as the constant function 1.
Measure on add_circle T
#
In this file we use the Haar measure on add_circle T
normalised to have total measure 1 (which is
not the same as the standard measure defined in topology.instances.add_circle
).
Haar measure on the additive circle, normalised to have total measure 1.
Instances for add_circle.haar_add_circle
The family of exponential monomials λ x, exp (2 π i n x / T)
, parametrized by n : ℤ
and
considered as bundled continuous maps from ℝ / ℤ • T
to ℂ
.
Equations
- fourier n = {to_fun := λ (x : add_circle T), ↑((n • x).to_circle), continuous_to_fun := _}
The subalgebra of C(add_circle T, ℂ)
generated by fourier n
for n ∈ ℤ
.
Equations
The subalgebra of C(add_circle T, ℂ)
generated by fourier n
for n ∈ ℤ
is in fact the
linear span of these functions.
The subalgebra of C(add_circle T, ℂ)
generated by fourier n
for n ∈ ℤ
is invariant under
complex conjugation.
The subalgebra of C(add_circle T, ℂ)
generated by fourier n
for n ∈ ℤ
separates points.
The subalgebra of C(add_circle T, ℂ)
generated by fourier n
for n ∈ ℤ
is dense.
The linear span of the monomials fourier n
is dense in C(add_circle T, ℂ)
.
The family of monomials fourier n
, parametrized by n : ℤ
and considered as
elements of the Lp
space of functions add_circle T → ℂ
.
For each 1 ≤ p < ∞
, the linear span of the monomials fourier n
is dense in
Lp ℂ p haar_circle
.
The monomials fourier n
are an orthonormal set with respect to normalised Haar measure.
The n
-th Fourier coefficient of a function add_circle T → E
, for E
a complete normed
ℂ
-vector space, defined as the integral over add_circle T
of fourier (-n) t • f t
.
Equations
- fourier_coeff f n = ∫ (t : add_circle T), ⇑(fourier (-n)) t • f t ∂add_circle.haar_add_circle
The Fourier coefficients of a function on add_circle T
can be computed as an integral
over [a, a + T]
, for any real a
.
For a function on ℝ
, the Fourier coefficients of f
on [a, b]
are defined as the
Fourier coefficients of the unique periodic function agreeing with f
on Ioc a b
.
Equations
- fourier_coeff_on hab f n = fourier_coeff (add_circle.lift_Ioc (b - a) a f) n
We define fourier_basis
to be a ℤ
-indexed Hilbert basis for Lp ℂ 2 haar_add_circle
,
which by definition is an isometric isomorphism from Lp ℂ 2 haar_add_circle
to ℓ²(ℤ, ℂ)
.
Equations
- fourier_basis = hilbert_basis.mk orthonormal_fourier fourier_basis._proof_2
The elements of the Hilbert basis fourier_basis
are the functions fourier_Lp 2
, i.e. the
monomials fourier n
on the circle considered as elements of L²
.
Under the isometric isomorphism fourier_basis
from Lp ℂ 2 haar_circle
to ℓ²(ℤ, ℂ)
, the
i
-th coefficient is fourier_coeff f i
, i.e., the integral over add_circle T
of
λ t, fourier (-i) t * f t
with respect to the Haar measure of total mass 1.
The Fourier series of an L2
function f
sums to f
, in the L²
space of add_circle T
.
Parseval's identity: for an L²
function f
on add_circle T
, the sum of the squared
norms of the Fourier coefficients equals the L²
norm of f
.
If the sequence of Fourier coefficients of f
is summable, then the Fourier series converges
uniformly to f
.
If the sequence of Fourier coefficients of f
is summable, then the Fourier series of f
converges everywhere pointwise to f
.
Express Fourier coefficients of f
on an interval in terms of those of its derivative.