Convergence in distribution #
We introduce a definition of convergence in distribution of random variables: this is the
weak convergence of the laws of the random variables. In Mathlib terms this is a Tendsto in the
ProbabilityMeasure type.
The definition assumes that the random variables are defined on the same probability space, which
is the most common setting in applications. Convergence in distribution for random variables
on different probability spaces can be talked about using the ProbabilityMeasure type directly.
Main definitions #
TendstoInDistribution X l Z μ: the sequence of random variablesX nconverges in distribution to the random variableZalong the filterlwith respect to the probability measureμ.
Main statements #
TendstoInDistribution.continuous_comp: Continuous mapping theorem. IfX ntends toZin distribution andgis continuous, theng ∘ X ntends tog ∘ Zin distribution.
Convergence in distribution of random variables.
This is the weak convergence of the laws of the random variables: Tendsto in the
ProbabilityMeasure type.
- forall_aemeasurable (i : ι) : AEMeasurable (X i) μ
- aemeasurable_limit : AEMeasurable Z μ
- tendsto : Filter.Tendsto (fun (n : ι) => ⟨Measure.map (X n) μ, ⋯⟩) l (nhds ⟨Measure.map Z μ, ⋯⟩)
Instances For
Continuous mapping theorem: if X n tends to Z in distribution and g is continuous,
then g ∘ X n tends to g ∘ Z in distribution.