Convergence in measure #
We define convergence in measure which is one of the many notions of convergence in probability.
A sequence of functions f
is said to converge in measure to some function g
if for all ε > 0
, the measure of the set {x | ε ≤ dist (f i x) (g x)}
tends to 0 as i
converges along some given filter l
.
Convergence in measure is most notably used in the formulation of the weak law of large numbers and is also useful in theorems such as the Vitali convergence theorem. This file provides some basic lemmas for working with convergence in measure and establishes some relations between convergence in measure and other notions of convergence.
Main definitions #
MeasureTheory.TendstoInMeasure (μ : Measure α) (f : ι → α → E) (g : α → E)
:f
converges inμ
-measure tog
.
Main results #
MeasureTheory.tendstoInMeasure_of_tendsto_ae
: convergence almost everywhere in a finite measure space implies convergence in measure.MeasureTheory.TendstoInMeasure.exists_seq_tendsto_ae
: iff
is a sequence of functions which converges in measure tog
, thenf
has a subsequence which convergence almost everywhere tog
.MeasureTheory.exists_seq_tendstoInMeasure_atTop_iff
: for a sequence of functionsf
, convergence in measure is equivalent to the fact that every subsequence has another subsequence that converges almost surely.MeasureTheory.tendstoInMeasure_of_tendsto_eLpNorm
: convergence in Lp implies convergence in measure.
A sequence of functions f
is said to converge in measure to some function g
if for all
ε > 0
, the measure of the set {x | ε ≤ dist (f i x) (g x)}
tends to 0 as i
converges along
some given filter l
.
Equations
Instances For
Auxiliary lemma for tendstoInMeasure_of_tendsto_ae
.
Convergence a.e. implies convergence in measure in a finite measure space.
Given a sequence of functions f
which converges in measure to g
,
seqTendstoAeSeqAux
is a sequence such that
∀ m ≥ seqTendstoAeSeqAux n, μ {x | 2⁻¹ ^ n ≤ dist (f m x) (g x)} ≤ 2⁻¹ ^ n
.
Equations
Instances For
Transformation of seqTendstoAeSeqAux
to makes sure it is strictly monotone.
Equations
- MeasureTheory.ExistsSeqTendstoAe.seqTendstoAeSeq hfg 0 = MeasureTheory.ExistsSeqTendstoAe.seqTendstoAeSeqAux hfg 0
- MeasureTheory.ExistsSeqTendstoAe.seqTendstoAeSeq hfg n.succ = MeasureTheory.ExistsSeqTendstoAe.seqTendstoAeSeqAux hfg (n + 1) ⊔ (MeasureTheory.ExistsSeqTendstoAe.seqTendstoAeSeq hfg n + 1)
Instances For
If f
is a sequence of functions which converges in measure to g
, then there exists a
subsequence of f
which converges a.e. to g
.
TendstoInMeasure
is equivalent to every subsequence having another subsequence
which converges almost surely.
The limit in measure is ae unique.
This lemma is superseded by MeasureTheory.tendstoInMeasure_of_tendsto_eLpNorm
where we
allow p = ∞
and only require AEStronglyMeasurable
.
This lemma is superseded by MeasureTheory.tendstoInMeasure_of_tendsto_eLpNorm
where we
allow p = ∞
.
See also MeasureTheory.tendstoInMeasure_of_tendsto_eLpNorm
which work for general
Lp-convergence for all p ≠ 0
.
Convergence in Lp implies convergence in measure.
Convergence in Lp implies convergence in measure.