Convergence in measure #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
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 #
measure_theory.tendsto_in_measure (μ : measure α) (f : ι → α → E) (g : α → E)
:f
converges inμ
-measure tog
.
Main results #
measure_theory.tendsto_in_measure_of_tendsto_ae
: convergence almost everywhere in a finite measure space implies convergence in measure.measure_theory.tendsto_in_measure.exists_seq_tendsto_ae
: iff
is a sequence of functions which converges in measure tog
, thenf
has a subsequence which convergence almost everywhere tog
.measure_theory.tendsto_in_measure_of_tendsto_snorm
: 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
- measure_theory.tendsto_in_measure μ f l g = ∀ (ε : ℝ), 0 < ε → filter.tendsto (λ (i : ι), ⇑μ {x : α | ε ≤ has_dist.dist (f i x) (g x)}) l (nhds 0)
Auxiliary lemma for tendsto_in_measure_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
,
seq_tendsto_ae_seq_aux
is a sequence such that
∀ m ≥ seq_tendsto_ae_seq_aux n, μ {x | 2⁻¹ ^ n ≤ dist (f m x) (g x)} ≤ 2⁻¹ ^ n
.
Equations
Transformation of seq_tendsto_ae_seq_aux
to makes sure it is strictly monotone.
Equations
- measure_theory.exists_seq_tendsto_ae.seq_tendsto_ae_seq hfg (n + 1) = linear_order.max (measure_theory.exists_seq_tendsto_ae.seq_tendsto_ae_seq_aux hfg (n + 1)) (measure_theory.exists_seq_tendsto_ae.seq_tendsto_ae_seq hfg n + 1)
- measure_theory.exists_seq_tendsto_ae.seq_tendsto_ae_seq hfg 0 = measure_theory.exists_seq_tendsto_ae.seq_tendsto_ae_seq_aux hfg 0
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
.
This lemma is superceded by measure_theory.tendsto_in_measure_of_tendsto_snorm
where we
allow p = ∞
and only require ae_strongly_measurable
.
This lemma is superceded by measure_theory.tendsto_in_measure_of_tendsto_snorm
where we
allow p = ∞
.
See also measure_theory.tendsto_in_measure_of_tendsto_snorm
which work for general
Lp-convergence for all p ≠ 0
.
Convergence in Lp implies convergence in measure.
Convergence in Lp implies convergence in measure.