Documentation

Mathlib.MeasureTheory.Measure.CharacteristicFunction

Characteristic Function of a Finite Measure #

This file defines the characteristic function of a finite measure on a topological vector space V.

The characteristic function of a finite measure P on V is the mapping W → ℂ, w => ∫ v, e (L v w) ∂P, where e is a continuous additive character and L : V →ₗ[ℝ] W →ₗ[ℝ] ℝ is a bilinear map.

A typical example is V = W = ℝ and L v w = v * w.

The integral is expressed as ∫ v, char he hL w v ∂P, where char he hL w is the bounded continuous function fun v ↦ e (L v w) and he, hL are continuity hypotheses on e and L.

Main definitions #

Main statements #

The bounded continuous map x ↦ exp (L x * I), for a continuous linear form L.

Equations
Instances For
    theorem MeasureTheory.ext_of_integral_char_eq {W : Type u_1} [AddCommGroup W] [Module W] [TopologicalSpace W] {e : AddChar Circle} {V : Type u_2} [AddCommGroup V] [Module V] [PseudoEMetricSpace V] [MeasurableSpace V] [BorelSpace V] [CompleteSpace V] [SecondCountableTopology V] {L : V →ₗ[] W →ₗ[] } (he : Continuous e) (he' : e 1) (hL' : ∀ (v : V), v 0L v 0) (hL : Continuous fun (p : V × W) => (L p.1) p.2) {P P' : Measure V} [IsFiniteMeasure P] [IsFiniteMeasure P'] (h : ∀ (w : W), (v : V), (BoundedContinuousFunction.char he hL w) v P = (v : V), (BoundedContinuousFunction.char he hL w) v P') :
    P = P'

    If the integrals of char with respect to two finite measures P and P' coincide, then P = P'.

    noncomputable def MeasureTheory.charFun {E : Type u_2} {mE : MeasurableSpace E} [Inner E] (μ : Measure E) (t : E) :

    The characteristic function of a measure in an inner product space.

    Equations
    Instances For
      theorem MeasureTheory.charFun_apply {E : Type u_2} {mE : MeasurableSpace E} {μ : Measure E} [Inner E] (t : E) :
      charFun μ t = (x : E), Complex.exp ((inner x t) * Complex.I) μ
      @[simp]

      charFun as the integral of a bounded continuous function.

      charFun is a Fourier integral for the inner product and the character probChar.

      charFun is a Fourier integral for the inner product and the character fourierChar.

      theorem MeasureTheory.charFun_map_smul {E : Type u_2} {mE : MeasurableSpace E} {μ : Measure E} [SeminormedAddCommGroup E] [InnerProductSpace E] [BorelSpace E] [SecondCountableTopology E] (r : ) (t : E) :
      charFun (Measure.map (fun (x : E) => r x) μ) t = charFun μ (r t)
      theorem MeasureTheory.charFun_map_mul {μ : Measure } (r t : ) :
      charFun (Measure.map (fun (x : ) => r * x) μ) t = charFun μ (r * t)
      theorem MeasureTheory.charFun_map_add_const {E : Type u_3} [MeasurableSpace E] {μ : Measure E} [NormedAddCommGroup E] [InnerProductSpace E] [BorelSpace E] (r t : E) :
      charFun (Measure.map (fun (x : E) => x + r) μ) t = charFun μ t * Complex.exp ((inner r t) * Complex.I)
      theorem MeasureTheory.charFun_map_const_add {E : Type u_3} [MeasurableSpace E] {μ : Measure E} [NormedAddCommGroup E] [InnerProductSpace E] [BorelSpace E] (r t : E) :
      charFun (Measure.map (fun (x : E) => r + x) μ) t = charFun μ t * Complex.exp ((inner r t) * Complex.I)

      If the characteristic functions charFun of two finite measures μ and ν on a complete second-countable inner product space coincide, then μ = ν.

      The characteristic function of a convolution of measures is the product of the respective characteristic functions.

      theorem MeasureTheory.charFun_prod {E : Type u_4} {F : Type u_5} [NormedAddCommGroup E] [NormedAddCommGroup F] [InnerProductSpace E] [InnerProductSpace F] {mE : MeasurableSpace E} {mF : MeasurableSpace F} {μ : Measure E} {ν : Measure F} [SFinite μ] [SFinite ν] (t : WithLp 2 (E × F)) :
      charFun (Measure.map (WithLp.toLp 2) (μ.prod ν)) t = charFun μ t.ofLp.1 * charFun ν t.ofLp.2

      The characteristic function of a product of measures is a product of characteristic functions. This is the version for Hilbert spaces, see charFunDual_prod for the Banach space version.

      The characteristic function of a measure is a product of characteristic functions if and only if it is a product measure. This is the version for Hilbert spaces, see charFunDual_eq_prod_iff for the Banach space version.

      theorem MeasureTheory.charFun_pi {ι : Type u_6} [Fintype ι] {E : ιType u_7} [(i : ι) → NormedAddCommGroup (E i)] [(i : ι) → InnerProductSpace (E i)] {mE : (i : ι) → MeasurableSpace (E i)} {μ : (i : ι) → Measure (E i)} [∀ (i : ι), SigmaFinite (μ i)] (t : PiLp 2 E) :
      charFun (Measure.map (WithLp.toLp 2) (Measure.pi μ)) t = i : ι, charFun (μ i) (t i)

      The characteristic function of a product of measures is a product of characteristic functions. This is the version for Hilbert spaces, see charFunDual_pi for the Banach space version.

      theorem MeasureTheory.charFun_eq_pi_iff {ι : Type u_6} [Fintype ι] {E : ιType u_7} [(i : ι) → NormedAddCommGroup (E i)] [(i : ι) → InnerProductSpace (E i)] {mE : (i : ι) → MeasurableSpace (E i)} [∀ (i : ι), CompleteSpace (E i)] [∀ (i : ι), SecondCountableTopology (E i)] [∀ (i : ι), BorelSpace (E i)] {μ : (i : ι) → Measure (E i)} {ν : Measure ((i : ι) → E i)} [∀ (i : ι), IsFiniteMeasure (μ i)] [IsFiniteMeasure ν] :
      (∀ (t : WithLp 2 ((i : ι) → E i)), charFun (Measure.map (WithLp.toLp 2) ν) t = i : ι, charFun (μ i) (t i)) ν = Measure.pi μ

      The characteristic function of a measure is a product of characteristic functions if and only if it is a product measure. This is the version for Hilbert spaces, see charFunDual_eq_pi_iff for the Banach space version.

      noncomputable def MeasureTheory.charFunDual {E : Type u_2} [NormedAddCommGroup E] [NormedSpace E] {mE : MeasurableSpace E} (μ : Measure E) (L : StrongDual E) :

      The characteristic function of a measure in a normed space, function from StrongDual ℝ E to with charFunDual μ L = ∫ v, exp (L v * I) ∂μ.

      Equations
      Instances For
        theorem MeasureTheory.charFunDual_map_add_const {E : Type u_2} [NormedAddCommGroup E] [NormedSpace E] {mE : MeasurableSpace E} {μ : Measure E} [BorelSpace E] (r : E) (L : StrongDual E) :
        charFunDual (Measure.map (fun (x : E) => x + r) μ) L = charFunDual μ L * Complex.exp ((L r) * Complex.I)
        theorem MeasureTheory.charFunDual_map_const_add {E : Type u_2} [NormedAddCommGroup E] [NormedSpace E] {mE : MeasurableSpace E} {μ : Measure E} [BorelSpace E] (r : E) (L : StrongDual E) :
        charFunDual (Measure.map (fun (x : E) => r + x) μ) L = charFunDual μ L * Complex.exp ((L r) * Complex.I)

        The characteristic function of a product of measures is a product of characteristic functions. This is the version for Banach spaces, see charFun_prod for the Hilbert space version.

        The characteristic function of a product of measures is a product of characteristic functions. This is charFunDual_prod for WithLp. See charFun_prod for the Hilbert space version.

        theorem MeasureTheory.charFunDual_pi {ι : Type u_4} [Fintype ι] [DecidableEq ι] {E : ιType u_5} [(i : ι) → NormedAddCommGroup (E i)] [(i : ι) → NormedSpace (E i)] {mE : (i : ι) → MeasurableSpace (E i)} {μ : (i : ι) → Measure (E i)} [∀ (i : ι), SigmaFinite (μ i)] (L : StrongDual ((i : ι) → E i)) :

        The characteristic function of a product of measures is a product of characteristic functions. This is the version for Banach spaces, see charFunDual_pi for the Hilbert space version.

        theorem MeasureTheory.charFunDual_pi' (p : ENNReal) [Fact (1 p)] {ι : Type u_4} [Fintype ι] [DecidableEq ι] {E : ιType u_5} [(i : ι) → NormedAddCommGroup (E i)] [(i : ι) → NormedSpace (E i)] {mE : (i : ι) → MeasurableSpace (E i)} {μ : (i : ι) → Measure (E i)} [∀ (i : ι), SigmaFinite (μ i)] (L : StrongDual (PiLp p E)) :

        The characteristic function of a product of measures is a product of characteristic functions. This is charFunDual_pi for PiLp. See charFunDual_pi for the Banach space version.

        If two finite measures have the same characteristic function, then they are equal.

        The characteristic function of a measure is a product of characteristic functions if and only if it is a product measure. This is the version for Banach spaces, see charFun_eq_prod_iff for the Hilbert space version.

        The characteristic function of a measure is a product of characteristic functions if and only if it is a product measure. This is charFunDual_eq_prod_iff for WithLp. See charFun_eq_prod_iff for the Hilbert space version.

        theorem MeasureTheory.charFunDual_eq_pi_iff {ι : Type u_4} [Fintype ι] [DecidableEq ι] {E : ιType u_5} [(i : ι) → NormedAddCommGroup (E i)] [(i : ι) → NormedSpace (E i)] {mE : (i : ι) → MeasurableSpace (E i)} [∀ (i : ι), BorelSpace (E i)] [∀ (i : ι), SecondCountableTopology (E i)] [∀ (i : ι), CompleteSpace (E i)] {μ : (i : ι) → Measure (E i)} {ν : Measure ((i : ι) → E i)} [∀ (i : ι), IsFiniteMeasure (μ i)] [IsFiniteMeasure ν] :
        (∀ (L : StrongDual ((i : ι) → E i)), charFunDual ν L = i : ι, charFunDual (μ i) (ContinuousLinearMap.comp L (ContinuousLinearMap.single E i))) ν = Measure.pi μ

        The characteristic function of a measure is a product of characteristic functions if and only if it is a product measure. This is the version for Banach spaces, see charFun_eq_pi_iff for the Hilbert space version.

        theorem MeasureTheory.charFunDual_eq_pi_iff' (p : ENNReal) [Fact (1 p)] {ι : Type u_4} [Fintype ι] [DecidableEq ι] {E : ιType u_5} [(i : ι) → NormedAddCommGroup (E i)] [(i : ι) → NormedSpace (E i)] {mE : (i : ι) → MeasurableSpace (E i)} [∀ (i : ι), BorelSpace (E i)] [∀ (i : ι), SecondCountableTopology (E i)] [∀ (i : ι), CompleteSpace (E i)] {μ : (i : ι) → Measure (E i)} {ν : Measure ((i : ι) → E i)} [∀ (i : ι), IsFiniteMeasure (μ i)] [IsFiniteMeasure ν] :
        (∀ (L : StrongDual (WithLp p ((i : ι) → E i))), charFunDual (Measure.map (WithLp.toLp p) ν) L = i : ι, charFunDual (μ i) (ContinuousLinearMap.comp L ((↑(PiLp.continuousLinearEquiv p E).symm).comp (ContinuousLinearMap.single E i)))) ν = Measure.pi μ

        The characteristic function of a measure is a product of characteristic functions if and only if it is a product measure. This is charFunDual_eq_pi_iff for PiLp. See charFun_eq_pi_iff for the Hilbert space version.

        The characteristic function of a convolution of measures is the product of the respective characteristic functions.