Egorov theorem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains the Egorov theorem which states that an almost everywhere convergent sequence on a finite measure space converges uniformly except on an arbitrarily small set. This theorem is useful for the Vitali convergence theorem as well as theorems regarding convergence in measure.
Main results #
measure_theory.egorov
: Egorov's theorem which shows that a sequence of almost everywhere convergent functions converges uniformly except on an arbitrarily small set.
Given a sequence of functions f
and a function g
, not_convergent_seq f g n j
is the
set of elements such that f k x
and g x
are separated by at least 1 / (n + 1)
for some
k ≥ j
.
This definition is useful for Egorov's theorem.
Equations
- measure_theory.egorov.not_convergent_seq f g n j = ⋃ (k : ι) (hk : j ≤ k), {x : α | 1 / (↑n + 1) < has_dist.dist (f k x) (g x)}
Given some ε > 0
, not_convergent_seq_lt_index
provides the index such that
not_convergent_seq
(intersected with a set of finite measure) has measure less than
ε * 2⁻¹ ^ n
.
This definition is useful for Egorov's theorem.
Equations
- measure_theory.egorov.not_convergent_seq_lt_index hε hf hg hsm hs hfg n = classical.some _
Given some ε > 0
, Union_not_convergent_seq
is the union of not_convergent_seq
with
specific indicies such that Union_not_convergent_seq
has measure less equal than ε
.
This definition is useful for Egorov's theorem.
Equations
- measure_theory.egorov.Union_not_convergent_seq hε hf hg hsm hs hfg = ⋃ (n : ℕ), s ∩ measure_theory.egorov.not_convergent_seq f g n (measure_theory.egorov.not_convergent_seq_lt_index _ hf hg hsm hs hfg n)
Egorov's theorem: If f : ι → α → β
is a sequence of strongly measurable functions that
converges to g : α → β
almost everywhere on a measurable set s
of finite measure,
then for all ε > 0
, there exists a subset t ⊆ s
such that μ t ≤ ε
and f
converges to g
uniformly on s \ t
. We require the index type ι
to be countable, and usually ι = ℕ
.
In other words, a sequence of almost everywhere convergent functions converges uniformly except on an arbitrarily small set.
Egorov's theorem for finite measure spaces.