The Fourier transform #
We set up the Fourier transform for complex-valued functions on finite-dimensional spaces.
Design choices #
In namespace VectorFourier, we define the Fourier integral in the following context:
๐is a commutative ring.VandWare๐-modules.eis a unitary additive character of๐, i.e. anAddChar ๐ Circle.ฮผis a measure onV.Lis a๐-bilinear formV ร W โ ๐.Eis a complete normedโ-vector space.
With these definitions, we define fourierIntegral to be the map from functions V โ E to
functions W โ E that sends f to
fun w โฆ โซ v in V, e (-L v w) โข f v โฮผ,
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.fourierChar, i.e. the character fun x โฆ exp ((2 * ฯ * x) * I) (for which we
introduced the notation ๐ in the scope FourierTransform).
Another familiar case (which generalizes the previous one) is when V = W is an inner product space
over โ and L is the scalar product. We introduce two notations ๐ for the Fourier transform in
this case and ๐โป f (v) = ๐ f (-v) for the inverse Fourier transform. These notations make
in particular sense for V = W = โ.
Main results #
At present the only nontrivial lemma we prove is fourierIntegral_continuous, 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.
Instances For
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.
In this section we assume ๐, V, W have topologies,
and L, e are continuous (but f needn't be).
This is used to ensure that e (-L v w) is (a.e. strongly) measurable. We could get away with
imposing only a measurable-space structure on ๐ (it doesn't have to be the Borel sigma-algebra of
a topology); but it seems hard to imagine cases where this extra generality would be useful, and
allowing it would complicate matters in the most important use cases.
For any w, the Fourier integral is convergent iff f is integrable.
The Fourier integral of an L^1 function is a continuous function.
Fubini's theorem for the Fourier integral.
This is the main technical step in proving both Parseval's identity and self-adjointness of the Fourier transform.
The Fourier transform satisfies โซ ๐ f * g = โซ f * ๐ g, i.e., it is self-adjoint.
Version where the multiplication is replaced by a general bilinear form M.
The Fourier transform satisfies โซ ๐ f * g = โซ f * ๐ g, i.e., it is self-adjoint.
The Fourier transform satisfies โซ ๐ f * conj g = โซ f * conj (๐โปยน g), which together
with the Fourier inversion theorem yields Plancherel's theorem. The stated version is more
convenient since it does only require integrability of f and g.
Version where the multiplication is replaced by a general bilinear form M.
Fourier theory for functions on ๐ #
The Fourier transform integral for f : ๐ โ E, with respect to the measure ฮผ and additive
character e.
Equations
- Fourier.fourierIntegral e ฮผ f w = VectorFourier.fourierIntegral e ฮผ (LinearMap.mul ๐ ๐) f w
Instances For
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 Fourier integral is well defined iff the function is integrable. Version with a general
continuous bilinear function L. For the specialization to the inner product in an inner product
space, see Real.fourierIntegral_convergent_iff.
Equations
- Real.instFourierTransform = { fourier := fun (f : V โ E) => VectorFourier.fourierIntegral Real.fourierChar MeasureTheory.volume (innerโ V) f }
Equations
- Real.instFourierTransformInv = { fourierInv := fun (f : V โ E) (w : V) => VectorFourier.fourierIntegral Real.fourierChar MeasureTheory.volume (-innerโ V) f w }
Alias of FourierTransform.fourier.
Equations
Instances For
Alias of FourierTransformInv.fourierInv.
Instances For
Alias of Real.fourier_eq.
Alias of Real.fourier_eq'.
Alias of Real.fourierInv_eq.
Alias of Real.fourierInv_eq'.
Alias of Real.fourier_comp_linearIsometry.
Alias of Real.fourierInv_eq_fourier_neg.
Alias of Real.fourierInv_eq_fourier_comp_neg.
Alias of Real.fourierInv_comm.
Alias of Real.fourierInv_comp_linearIsometry.
Alias of Real.fourier_real_eq.
Alias of Real.fourier_real_eq_integral_exp_smul.
Alias of Real.fourier_continuousLinearMap_apply.