Documentation

Mathlib.Probability.Independence.CharacteristicFunction

Links between independence and characteristic function #

Two random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. More specifically, prove this in Hilbert spaces for two variables and a finite family of variables. We prove the analoguous statemens in Banach spaces, with an arbitrary Lp norm, for the dual characteristic function.

Two random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. This is the version for Hilbert spaces, see indepFun_iff_charFunDual_prod for the Banach space version.

Two random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. This is the version for Banach spaces, see indepFun_iff_charFun_prod for the Hilbert space version.

Two random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. This is indepFun_iff_charFunDual_prod for WithLp. See indepFun_iff_charFun_prod for the Hilbert space version.

theorem ProbabilityTheory.iIndepFun_iff_charFun_pi {Ω : Type u_1} { : MeasurableSpace Ω} {P : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure P] {ι : Type u_2} [Fintype ι] {E : ιType u_3} {mE : (i : ι) → MeasurableSpace (E i)} [(i : ι) → NormedAddCommGroup (E i)] [∀ (i : ι), CompleteSpace (E i)] [∀ (i : ι), BorelSpace (E i)] [∀ (i : ι), SecondCountableTopology (E i)] {X : (i : ι) → ΩE i} [(i : ι) → InnerProductSpace (E i)] (hX : ∀ (i : ι), AEMeasurable (X i) P) :
iIndepFun X P ∀ (t : WithLp 2 ((x : ι) → E x)), MeasureTheory.charFun (MeasureTheory.Measure.map (fun (ω : Ω) => WithLp.toLp 2 fun (x : ι) => X x ω) P) t = i : ι, MeasureTheory.charFun (MeasureTheory.Measure.map (X i) P) (t i)

A finite number of random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. This is the version for Hilbert spaces, see iIndepFun_iff_charFunDual_pi for the Hilbert space version.

theorem ProbabilityTheory.iIndepFun_iff_charFunDual_pi {Ω : Type u_1} { : MeasurableSpace Ω} {P : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure P] {ι : Type u_2} [Fintype ι] {E : ιType u_3} {mE : (i : ι) → MeasurableSpace (E i)} [(i : ι) → NormedAddCommGroup (E i)] [∀ (i : ι), CompleteSpace (E i)] [∀ (i : ι), BorelSpace (E i)] [∀ (i : ι), SecondCountableTopology (E i)] {X : (i : ι) → ΩE i} [(i : ι) → NormedSpace (E i)] [DecidableEq ι] (hX : ∀ (i : ι), AEMeasurable (X i) P) :

A finite number of random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. This is the version for Banach spaces, see iIndepFun_iff_charFun_pi for the Hilbert space version.

theorem ProbabilityTheory.iIndepFun_iff_charFunDual_pi' {Ω : Type u_1} { : MeasurableSpace Ω} {P : MeasureTheory.Measure Ω} (p : ENNReal) [Fact (1 p)] [MeasureTheory.IsProbabilityMeasure P] {ι : Type u_2} [Fintype ι] {E : ιType u_3} {mE : (i : ι) → MeasurableSpace (E i)} [(i : ι) → NormedAddCommGroup (E i)] [∀ (i : ι), CompleteSpace (E i)] [∀ (i : ι), BorelSpace (E i)] [∀ (i : ι), SecondCountableTopology (E i)] {X : (i : ι) → ΩE i} [(i : ι) → NormedSpace (E i)] [DecidableEq ι] (hX : ∀ (i : ι), AEMeasurable (X i) P) :

A finite number of random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. This is iIndepFun_iff_charFunDual_pi for WithLp. See iIndepFun_iff_charFun_pi for the Hilbert space version.