Documentation

Mathlib.Probability.IdentDistrib

Identically distributed random variables #

Two random variables defined on two (possibly different) probability spaces but taking value in the same space are identically distributed if their distributions (i.e., the image probability measures on the target space) coincide. We define this concept and establish its basic properties in this file.

Main definitions and results #

There are two main kinds of lemmas, under the assumption that f and g are identically distributed: lemmas saying that two quantities computed for f and g are the same, and lemmas saying that if f has some property then g also has it. The first kind is registered as IdentDistrib.foo_fst, the second one as IdentDistrib.foo_snd (in the latter case, to deduce a property of f from one of g, use h.symm.foo_snd where h : IdentDistrib f g μ ν). For instance:

We also register several dot notation shortcuts for convenience. For instance, if h : IdentDistrib f g μ ν, then h.sq states that f^2 and g^2 are identically distributed, and h.norm states that ‖f‖ and ‖g‖ are identically distributed, and so on.

structure ProbabilityTheory.IdentDistrib {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] (f : αγ) (g : βγ) (μ : autoParam (MeasureTheory.Measure α) _auto✝) (ν : autoParam (MeasureTheory.Measure β) _auto✝) :

Two functions defined on two (possibly different) measure spaces are identically distributed if their image measures coincide. This only makes sense when the functions are ae measurable (as otherwise the image measures are not defined), so we require this as well in the definition.

Instances For
    theorem ProbabilityTheory.IdentDistrib.refl {α : Type u_1} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {f : αγ} (hf : AEMeasurable f μ) :
    theorem ProbabilityTheory.IdentDistrib.symm {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    theorem ProbabilityTheory.IdentDistrib.trans {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_4} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] [MeasurableSpace δ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} {ρ : MeasureTheory.Measure δ} {h : δγ} (h₁ : ProbabilityTheory.IdentDistrib f g μ ν) (h₂ : ProbabilityTheory.IdentDistrib g h ν ρ) :
    theorem ProbabilityTheory.IdentDistrib.comp_of_aemeasurable {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_4} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] [MeasurableSpace δ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} {u : γδ} (h : ProbabilityTheory.IdentDistrib f g μ ν) (hu : AEMeasurable u (MeasureTheory.Measure.map f μ)) :
    theorem ProbabilityTheory.IdentDistrib.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_4} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] [MeasurableSpace δ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} {u : γδ} (h : ProbabilityTheory.IdentDistrib f g μ ν) (hu : Measurable u) :
    theorem ProbabilityTheory.IdentDistrib.of_ae_eq {α : Type u_1} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {f : αγ} {g : αγ} (hf : AEMeasurable f μ) (heq : f =ᶠ[MeasureTheory.Measure.ae μ] g) :
    theorem ProbabilityTheory.IdentDistrib.measure_mem_eq {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} (h : ProbabilityTheory.IdentDistrib f g μ ν) {s : Set γ} (hs : MeasurableSet s) :
    μ (f ⁻¹' s) = ν (g ⁻¹' s)
    theorem ProbabilityTheory.IdentDistrib.measure_preimage_eq {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} (h : ProbabilityTheory.IdentDistrib f g μ ν) {s : Set γ} (hs : MeasurableSet s) :
    μ (f ⁻¹' s) = ν (g ⁻¹' s)

    Alias of ProbabilityTheory.IdentDistrib.measure_mem_eq.

    theorem ProbabilityTheory.IdentDistrib.ae_snd {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} (h : ProbabilityTheory.IdentDistrib f g μ ν) {p : γProp} (pmeas : MeasurableSet {x : γ | p x}) (hp : ∀ᵐ (x : α) ∂μ, p (f x)) :
    ∀ᵐ (x : β) ∂ν, p (g x)
    theorem ProbabilityTheory.IdentDistrib.ae_mem_snd {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} (h : ProbabilityTheory.IdentDistrib f g μ ν) {t : Set γ} (tmeas : MeasurableSet t) (ht : ∀ᵐ (x : α) ∂μ, f x t) :
    ∀ᵐ (x : β) ∂ν, g x t

    In a second countable topology, the first function in an identically distributed pair is a.e. strongly measurable. So is the second function, but use h.symm.aestronglyMeasurable_fst as h.aestronglyMeasurable_snd has a different meaning.

    If f and g are identically distributed and f is a.e. strongly measurable, so is g.

    theorem ProbabilityTheory.IdentDistrib.lintegral_eq {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [MeasurableSpace β] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αENNReal} {g : βENNReal} (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    ∫⁻ (x : α), f xμ = ∫⁻ (x : β), g xν
    theorem ProbabilityTheory.IdentDistrib.integral_eq {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [NormedAddCommGroup γ] [NormedSpace γ] [BorelSpace γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    ∫ (x : α), f xμ = ∫ (x : β), g xν
    theorem ProbabilityTheory.IdentDistrib.memℒp_snd {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [NormedAddCommGroup γ] [BorelSpace γ] {p : ENNReal} (h : ProbabilityTheory.IdentDistrib f g μ ν) (hf : MeasureTheory.Memℒp f p μ) :
    theorem ProbabilityTheory.IdentDistrib.norm {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [NormedAddCommGroup γ] [BorelSpace γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x) (fun (x : β) => g x) μ ν
    theorem ProbabilityTheory.IdentDistrib.nnnorm {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [NormedAddCommGroup γ] [BorelSpace γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x‖₊) (fun (x : β) => g x‖₊) μ ν
    theorem ProbabilityTheory.IdentDistrib.pow {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Pow γ ] [MeasurablePow γ ] (h : ProbabilityTheory.IdentDistrib f g μ ν) {n : } :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x ^ n) (fun (x : β) => g x ^ n) μ ν
    theorem ProbabilityTheory.IdentDistrib.sq {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Pow γ ] [MeasurablePow γ ] (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x ^ 2) (fun (x : β) => g x ^ 2) μ ν
    theorem ProbabilityTheory.IdentDistrib.coe_nnreal_ennreal {α : Type u_1} {β : Type u_2} [MeasurableSpace α] [MeasurableSpace β] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αNNReal} {g : βNNReal} (h : ProbabilityTheory.IdentDistrib f g μ ν) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => (f x)) (fun (x : β) => (g x)) μ ν
    theorem ProbabilityTheory.IdentDistrib.add_const {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Add γ] [MeasurableAdd γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x + c) (fun (x : β) => g x + c) μ ν
    theorem ProbabilityTheory.IdentDistrib.mul_const {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Mul γ] [MeasurableMul γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x * c) (fun (x : β) => g x * c) μ ν
    theorem ProbabilityTheory.IdentDistrib.const_add {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Add γ] [MeasurableAdd γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => c + f x) (fun (x : β) => c + g x) μ ν
    theorem ProbabilityTheory.IdentDistrib.const_mul {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Mul γ] [MeasurableMul γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => c * f x) (fun (x : β) => c * g x) μ ν
    theorem ProbabilityTheory.IdentDistrib.sub_const {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Sub γ] [MeasurableSub γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x - c) (fun (x : β) => g x - c) μ ν
    theorem ProbabilityTheory.IdentDistrib.div_const {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Div γ] [MeasurableDiv γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => f x / c) (fun (x : β) => g x / c) μ ν
    theorem ProbabilityTheory.IdentDistrib.const_sub {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Sub γ] [MeasurableSub γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => c - f x) (fun (x : β) => c - g x) μ ν
    theorem ProbabilityTheory.IdentDistrib.const_div {α : Type u_1} {β : Type u_2} {γ : Type u_3} [MeasurableSpace α] [MeasurableSpace β] [MeasurableSpace γ] {μ : MeasureTheory.Measure α} {ν : MeasureTheory.Measure β} {f : αγ} {g : βγ} [Div γ] [MeasurableDiv γ] (h : ProbabilityTheory.IdentDistrib f g μ ν) (c : γ) :
    ProbabilityTheory.IdentDistrib (fun (x : α) => c / f x) (fun (x : β) => c / g x) μ ν
    theorem ProbabilityTheory.Memℒp.uniformIntegrable_of_identDistrib_aux {α : Type u_1} [MeasurableSpace α] {E : Type u_5} [MeasurableSpace E] [NormedAddCommGroup E] [BorelSpace E] {μ : MeasureTheory.Measure α} [MeasureTheory.IsFiniteMeasure μ] {ι : Type u_6} {f : ιαE} {j : ι} {p : ENNReal} (hp : 1 p) (hp' : p ) (hℒp : MeasureTheory.Memℒp (f j) p μ) (hfmeas : ∀ (i : ι), MeasureTheory.StronglyMeasurable (f i)) (hf : ∀ (i : ι), ProbabilityTheory.IdentDistrib (f i) (f j) μ μ) :

    This lemma is superseded by Memℒp.uniformIntegrable_of_identDistrib which only requires AEStronglyMeasurable.

    theorem ProbabilityTheory.Memℒp.uniformIntegrable_of_identDistrib {α : Type u_1} [MeasurableSpace α] {E : Type u_5} [MeasurableSpace E] [NormedAddCommGroup E] [BorelSpace E] {μ : MeasureTheory.Measure α} [MeasureTheory.IsFiniteMeasure μ] {ι : Type u_6} {f : ιαE} {j : ι} {p : ENNReal} (hp : 1 p) (hp' : p ) (hℒp : MeasureTheory.Memℒp (f j) p μ) (hf : ∀ (i : ι), ProbabilityTheory.IdentDistrib (f i) (f j) μ μ) :

    A sequence of identically distributed Lᵖ functions is p-uniformly integrable.