Sequence of measurable functions associated to a sequence of a.e.-measurable functions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define here tools to prove statements about limits (infi, supr...) of sequences of
ae_measurable
functions.
Given a sequence of a.e.-measurable functions f : ι → α → β
with hypothesis
hf : ∀ i, ae_measurable (f i) μ
, and a pointwise property p : α → (ι → β) → Prop
such that we
have hp : ∀ᵐ x ∂μ, p x (λ n, f n x)
, we define a sequence of measurable functions ae_seq hf p
and a measurable set ae_seq_set hf p
, such that
μ (ae_seq_set hf p)ᶜ = 0
x ∈ ae_seq_set hf p → ∀ i : ι, ae_seq hf hp i x = f i x
x ∈ ae_seq_set hf p → p x (λ n, f n x)
If we have the additional hypothesis ∀ᵐ x ∂μ, p x (λ n, f n x)
, this is a measurable set
whose complement has measure 0 such that for all x ∈ ae_seq_set
, f i x
is equal to
(hf i).mk (f i) x
for all i
and we have the pointwise property p x (λ n, f n x)
.
Equations
- ae_seq_set hf p = (measure_theory.to_measurable μ {x : α | (∀ (i : ι), f i x = ae_measurable.mk (f i) _ x) ∧ p x (λ (n : ι), f n x)}ᶜ)ᶜ
A sequence of measurable functions that are equal to f
and verify property p
on the
measurable set ae_seq_set hf p
.
Equations
- ae_seq hf p = λ (i : ι) (x : α), ite (x ∈ ae_seq_set hf p) (ae_measurable.mk (f i) _ x) _.some