mathlib3 documentation

measure_theory.function.strongly_measurable.basic

Strongly measurable and finitely strongly measurable functions #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

A function f is said to be strongly measurable if f is the sequential limit of simple functions. It is said to be finitely strongly measurable with respect to a measure μ if the supports of those simple functions have finite measure. We also provide almost everywhere versions of these notions.

Almost everywhere strongly measurable functions form the largest class of functions that can be integrated using the Bochner integral.

If the target space has a second countable topology, strongly measurable and measurable are equivalent.

If the measure is sigma-finite, strongly measurable and finitely strongly measurable are equivalent.

The main property of finitely strongly measurable functions is fin_strongly_measurable.exists_set_sigma_finite: there exists a measurable set t such that the function is supported on t and μ.restrict t is sigma-finite. As a consequence, we can prove some results for those functions as if the measure was sigma-finite.

Main definitions #

Main statements #

We provide a solid API for strongly measurable functions, and for almost everywhere strongly measurable functions, as a basis for the Bochner integral.

References #

@[class]
structure second_countable_topology_either (α : Type u_1) (β : Type u_2) [topological_space α] [topological_space β] :
Prop

The typeclass second_countable_topology_either α β registers the fact that at least one of the two spaces has second countable topology. This is the right assumption to ensure that continuous maps from α to β are strongly measurable.

Instances of this typeclass
def measure_theory.strongly_measurable {α : Type u_1} {β : Type u_2} [topological_space β] [measurable_space α] (f : α β) :
Prop

A function is strongly_measurable if it is the limit of simple functions.

Equations
def measure_theory.fin_strongly_measurable {α : Type u_1} {β : Type u_2} [topological_space β] [has_zero β] {m0 : measurable_space α} (f : α β) (μ : measure_theory.measure α) :
Prop

A function is fin_strongly_measurable with respect to a measure if it is the limit of simple functions with support with finite measure.

Equations
def measure_theory.ae_strongly_measurable {α : Type u_1} {β : Type u_2} [topological_space β] {m0 : measurable_space α} (f : α β) (μ : measure_theory.measure α) :
Prop

A function is ae_strongly_measurable with respect to a measure μ if it is almost everywhere equal to the limit of a sequence of simple functions.

Equations
def measure_theory.ae_fin_strongly_measurable {α : Type u_1} {β : Type u_2} [topological_space β] [has_zero β] {m0 : measurable_space α} (f : α β) (μ : measure_theory.measure α) :
Prop

A function is ae_fin_strongly_measurable with respect to a measure if it is almost everywhere equal to the limit of a sequence of simple functions with support with finite measure.

Equations

Strongly measurable functions #

theorem measure_theory.strongly_measurable_const {α : Type u_1} {β : Type u_2} {m : measurable_space α} [topological_space β] {b : β} :
theorem measure_theory.strongly_measurable_const' {α : Type u_1} {β : Type u_2} {m : measurable_space α} [topological_space β] {f : α β} (hf : (x y : α), f x = f y) :

A version of strongly_measurable_const that assumes f x = f y for all x, y. This version works for functions between empty types.

@[protected]

A sequence of simple functions such that ∀ x, tendsto (λ n, hf.approx n x) at_top (𝓝 (f x)). That property is given by strongly_measurable.tendsto_approx.

Equations
@[protected]
theorem measure_theory.strongly_measurable.tendsto_approx {α : Type u_1} {β : Type u_2} {f : α β} [topological_space β] {m : measurable_space α} (hf : measure_theory.strongly_measurable f) (x : α) :
filter.tendsto (λ (n : ), (hf.approx n) x) filter.at_top (nhds (f x))

Similar to strongly_measurable.approx, but enforces that the norm of every function in the sequence is less than c everywhere. If ‖f x‖ ≤ c this sequence of simple functions verifies tendsto (λ n, hf.approx_bounded n x) at_top (𝓝 (f x)).

Equations
theorem measure_theory.strongly_measurable.tendsto_approx_bounded_ae {α : Type u_1} {β : Type u_2} {f : α β} [normed_add_comm_group β] [normed_space β] {m m0 : measurable_space α} {μ : measure_theory.measure α} (hf : measure_theory.strongly_measurable f) {c : } (hf_bound : ∀ᵐ (x : α) μ, f x c) :
∀ᵐ (x : α) μ, filter.tendsto (λ (n : ), (hf.approx_bounded c n) x) filter.at_top (nhds (f x))
theorem measure_theory.strongly_measurable.norm_approx_bounded_le {α : Type u_1} {β : Type u_2} {f : α β} [seminormed_add_comm_group β] [normed_space β] {m : measurable_space α} {c : } (hf : measure_theory.strongly_measurable f) (hc : 0 c) (n : ) (x : α) :
theorem strongly_measurable_bot_iff {α : Type u_1} {β : Type u_2} {f : α β} [topological_space β] [nonempty β] [t2_space β] :
measure_theory.strongly_measurable f (c : β), f = λ (_x : α), c
@[protected]

If the measure is sigma-finite, all strongly measurable functions are fin_strongly_measurable.

@[protected]

A strongly measurable function is measurable.

@[protected]

A strongly measurable function is almost everywhere measurable.

theorem continuous.comp_strongly_measurable {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} [topological_space β] [topological_space γ] {g : β γ} {f : α β} (hg : continuous g) (hf : measure_theory.strongly_measurable f) :
measure_theory.strongly_measurable (λ (x : α), g (f x))
@[protected]
@[protected]
theorem measure_theory.strongly_measurable.prod_mk {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} [topological_space β] [topological_space γ] {f : α β} {g : α γ} (hf : measure_theory.strongly_measurable f) (hg : measure_theory.strongly_measurable g) :
measure_theory.strongly_measurable (λ (x : α), (f x, g x))
theorem measure_theory.strongly_measurable.of_uncurry_right {α : Type u_1} {β : Type u_2} {γ : Type u_3} [topological_space β] {mα : measurable_space α} {mγ : measurable_space γ} {f : α γ β} (hf : measure_theory.strongly_measurable (function.uncurry f)) {y : γ} :
@[protected]
theorem measure_theory.strongly_measurable.vadd {α : Type u_1} {β : Type u_2} {mα : measurable_space α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_vadd 𝕜 β] [has_continuous_vadd 𝕜 β] {f : α 𝕜} {g : α β} (hf : measure_theory.strongly_measurable f) (hg : measure_theory.strongly_measurable g) :
@[protected]
theorem measure_theory.strongly_measurable.smul {α : Type u_1} {β : Type u_2} {mα : measurable_space α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_smul 𝕜 β] [has_continuous_smul 𝕜 β] {f : α 𝕜} {g : α β} (hf : measure_theory.strongly_measurable f) (hg : measure_theory.strongly_measurable g) :
@[protected]
theorem measure_theory.strongly_measurable.const_smul {α : Type u_1} {β : Type u_2} {f : α β} {mα : measurable_space α} [topological_space β] {𝕜 : Type u_3} [has_smul 𝕜 β] [has_continuous_const_smul 𝕜 β] (hf : measure_theory.strongly_measurable f) (c : 𝕜) :
@[protected]
theorem measure_theory.strongly_measurable.const_smul' {α : Type u_1} {β : Type u_2} {f : α β} {mα : measurable_space α} [topological_space β] {𝕜 : Type u_3} [has_smul 𝕜 β] [has_continuous_const_smul 𝕜 β] (hf : measure_theory.strongly_measurable f) (c : 𝕜) :
@[protected]
theorem measure_theory.strongly_measurable.smul_const {α : Type u_1} {β : Type u_2} {mα : measurable_space α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_smul 𝕜 β] [has_continuous_smul 𝕜 β] {f : α 𝕜} (hf : measure_theory.strongly_measurable f) (c : β) :
@[protected]
theorem measure_theory.strongly_measurable.vadd_const {α : Type u_1} {β : Type u_2} {mα : measurable_space α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_vadd 𝕜 β] [has_continuous_vadd 𝕜 β] {f : α 𝕜} (hf : measure_theory.strongly_measurable f) (c : β) :
theorem strongly_measurable_const_smul_iff₀ {α : Type u_1} {β : Type u_2} {f : α β} {G₀ : Type u_7} [topological_space β] [group_with_zero G₀] [mul_action G₀ β] [has_continuous_const_smul G₀ β] {m : measurable_space α} {c : G₀} (hc : c 0) :

Big operators: and #

theorem list.strongly_measurable_sum {α : Type u_1} {M : Type u_5} [add_monoid M] [topological_space M] [has_continuous_add M] {m : measurable_space α} (l : list M)) (hl : (f : α M), f l measure_theory.strongly_measurable f) :
measure_theory.strongly_measurable (λ (x : α), (list.map (λ (f : α M), f x) l).sum)
theorem list.strongly_measurable_prod {α : Type u_1} {M : Type u_5} [monoid M] [topological_space M] [has_continuous_mul M] {m : measurable_space α} (l : list M)) (hl : (f : α M), f l measure_theory.strongly_measurable f) :
measure_theory.strongly_measurable (λ (x : α), (list.map (λ (f : α M), f x) l).prod)
theorem multiset.strongly_measurable_sum {α : Type u_1} {M : Type u_5} [add_comm_monoid M] [topological_space M] [has_continuous_add M] {m : measurable_space α} (s : multiset M)) (hs : (f : α M), f s measure_theory.strongly_measurable f) :
measure_theory.strongly_measurable (λ (x : α), (multiset.map (λ (f : α M), f x) s).sum)
theorem multiset.strongly_measurable_prod {α : Type u_1} {M : Type u_5} [comm_monoid M] [topological_space M] [has_continuous_mul M] {m : measurable_space α} (s : multiset M)) (hs : (f : α M), f s measure_theory.strongly_measurable f) :
measure_theory.strongly_measurable (λ (x : α), (multiset.map (λ (f : α M), f x) s).prod)
theorem finset.strongly_measurable_sum' {α : Type u_1} {M : Type u_5} [add_comm_monoid M] [topological_space M] [has_continuous_add M] {m : measurable_space α} {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.strongly_measurable (f i)) :
theorem finset.strongly_measurable_prod' {α : Type u_1} {M : Type u_5} [comm_monoid M] [topological_space M] [has_continuous_mul M] {m : measurable_space α} {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.strongly_measurable (f i)) :
theorem finset.strongly_measurable_prod {α : Type u_1} {M : Type u_5} [comm_monoid M] [topological_space M] [has_continuous_mul M] {m : measurable_space α} {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.strongly_measurable (f i)) :
measure_theory.strongly_measurable (λ (a : α), s.prod (λ (i : ι), f i a))
theorem finset.strongly_measurable_sum {α : Type u_1} {M : Type u_5} [add_comm_monoid M] [topological_space M] [has_continuous_add M] {m : measurable_space α} {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.strongly_measurable (f i)) :
measure_theory.strongly_measurable (λ (a : α), s.sum (λ (i : ι), f i a))

The range of a strongly measurable function is separable.

In a space with second countable topology, measurable implies strongly measurable.

In a space with second countable topology, strongly measurable and measurable are equivalent.

A function is strongly measurable if and only if it is measurable and has separable range.

A continuous function is strongly measurable when either the source space or the target space is second-countable.

If g is a topological embedding, then f is strongly measurable iff g ∘ f is.

theorem strongly_measurable_of_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_3} {m : measurable_space α} [topological_space β] [topological_space.pseudo_metrizable_space β] (u : filter ι) [u.ne_bot] [u.is_countably_generated] {f : ι α β} {g : α β} (hf : (i : ι), measure_theory.strongly_measurable (f i)) (lim : filter.tendsto f u (nhds g)) :

A sequential limit of strongly measurable functions is strongly measurable.

@[protected]
@[protected]
theorem measure_theory.strongly_measurable.ite {α : Type u_1} {β : Type u_2} {f g : α β} {m : measurable_space α} [topological_space β] {p : α Prop} {_x : decidable_pred p} (hp : measurable_set {a : α | p a}) (hf : measure_theory.strongly_measurable f) (hg : measure_theory.strongly_measurable g) :
measure_theory.strongly_measurable (λ (x : α), ite (p x) (f x) (g x))

this is slightly different from strongly_measurable.piecewise. It can be used to show strongly_measurable (ite (x=0) 0 1) by exact strongly_measurable.ite (measurable_set_singleton 0) strongly_measurable_const strongly_measurable_const, but replacing strongly_measurable.ite by strongly_measurable.piecewise in that example proof does not work.

@[protected]
theorem measurable_embedding.exists_strongly_measurable_extend {α : Type u_1} {β : Type u_2} {γ : Type u_3} {f : α β} {g : α γ} {mα : measurable_space α} {mγ : measurable_space γ} [topological_space β] (hg : measurable_embedding g) (hf : measure_theory.strongly_measurable f) (hne : γ nonempty β) :
theorem measure_theory.strongly_measurable.strongly_measurable_in_set {α : Type u_1} {β : Type u_2} {m : measurable_space α} [topological_space β] [has_zero β] {s : set α} {f : α β} (hs : measurable_set s) (hf : measure_theory.strongly_measurable f) (hf_zero : (x : α), x s f x = 0) :
(fs : measure_theory.simple_func α β), ( (x : α), filter.tendsto (λ (n : ), (fs n) x) filter.at_top (nhds (f x))) (x : α), x s (n : ), (fs n) x = 0
theorem measure_theory.strongly_measurable.strongly_measurable_of_measurable_space_le_on {α : Type u_1} {E : Type u_2} {m m₂ : measurable_space α} [topological_space E] [has_zero E] {s : set α} {f : α E} (hs_m : measurable_set s) (hs : (t : set α), measurable_set (s t) measurable_set (s t)) (hf : measure_theory.strongly_measurable f) (hf_zero : (x : α), x s f x = 0) :

If the restriction to a set s of a σ-algebra m is included in the restriction to s of another σ-algebra m₂ (hypothesis hs), the set s is m measurable and a function f supported on s is m-strongly-measurable, then f is also m₂-strongly-measurable.

theorem measure_theory.strongly_measurable.exists_spanning_measurable_set_norm_le {α : Type u_1} {β : Type u_2} {f : α β} [seminormed_add_comm_group β] {m m0 : measurable_space α} (hm : m m0) (hf : measure_theory.strongly_measurable f) (μ : measure_theory.measure α) [measure_theory.sigma_finite (μ.trim hm)] :
(s : set α), ( (n : ), measurable_set (s n) μ (s n) < (x : α), x s n f x n) ( (i : ), s i) = set.univ

If a function f is strongly measurable w.r.t. a sub-σ-algebra m and the measure is σ-finite on m, then there exists spanning measurable sets with finite measure on which f has bounded norm. In particular, f is integrable on each of those sets.

Finitely strongly measurable functions #

@[protected]

A sequence of simple functions such that ∀ x, tendsto (λ n, hf.approx n x) at_top (𝓝 (f x)) and ∀ n, μ (support (hf.approx n)) < ∞. These properties are given by fin_strongly_measurable.tendsto_approx and fin_strongly_measurable.fin_support_approx.

Equations
@[protected]
theorem measure_theory.fin_strongly_measurable.tendsto_approx {α : Type u_1} {β : Type u_2} {m0 : measurable_space α} {μ : measure_theory.measure α} {f : α β} [has_zero β] [topological_space β] (hf : measure_theory.fin_strongly_measurable f μ) (x : α) :
filter.tendsto (λ (n : ), (hf.approx n) x) filter.at_top (nhds (f x))
@[protected]

A finitely strongly measurable function is measurable.

@[protected]

Almost everywhere strongly measurable functions #

@[protected]
noncomputable def measure_theory.ae_strongly_measurable.mk {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] (f : α β) (hf : measure_theory.ae_strongly_measurable f μ) :
α β

A strongly_measurable function such that f =ᵐ[μ] hf.mk f. See lemmas strongly_measurable_mk and ae_eq_mk.

Equations
theorem continuous.comp_ae_strongly_measurable {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] [topological_space γ] {g : β γ} {f : α β} (hg : continuous g) (hf : measure_theory.ae_strongly_measurable f μ) :
measure_theory.ae_strongly_measurable (λ (x : α), g (f x)) μ

The composition of a continuous function and an ae strongly measurable function is ae strongly measurable.

A continuous function from α to β is ae strongly measurable when one of the two spaces is second countable.

@[protected]
theorem measure_theory.ae_strongly_measurable.prod_mk {α : Type u_1} {β : Type u_2} {γ : Type u_3} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] [topological_space γ] {f : α β} {g : α γ} (hf : measure_theory.ae_strongly_measurable f μ) (hg : measure_theory.ae_strongly_measurable g μ) :
measure_theory.ae_strongly_measurable (λ (x : α), (f x, g x)) μ

In a space with second countable topology, measurable implies ae strongly measurable.

@[protected]
@[protected]
@[protected]
@[protected]
@[protected]
theorem measure_theory.ae_strongly_measurable.smul {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_smul 𝕜 β] [has_continuous_smul 𝕜 β] {f : α 𝕜} {g : α β} (hf : measure_theory.ae_strongly_measurable f μ) (hg : measure_theory.ae_strongly_measurable g μ) :
measure_theory.ae_strongly_measurable (λ (x : α), f x g x) μ
@[protected]
theorem measure_theory.ae_strongly_measurable.vadd {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_vadd 𝕜 β] [has_continuous_vadd 𝕜 β] {f : α 𝕜} {g : α β} (hf : measure_theory.ae_strongly_measurable f μ) (hg : measure_theory.ae_strongly_measurable g μ) :
@[protected]
@[protected]
theorem measure_theory.ae_strongly_measurable.const_smul' {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {f : α β} {𝕜 : Type u_3} [has_smul 𝕜 β] [has_continuous_const_smul 𝕜 β] (hf : measure_theory.ae_strongly_measurable f μ) (c : 𝕜) :
@[protected]
theorem measure_theory.ae_strongly_measurable.vadd_const {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_vadd 𝕜 β] [has_continuous_vadd 𝕜 β] {f : α 𝕜} (hf : measure_theory.ae_strongly_measurable f μ) (c : β) :
@[protected]
theorem measure_theory.ae_strongly_measurable.smul_const {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {𝕜 : Type u_3} [topological_space 𝕜] [has_smul 𝕜 β] [has_continuous_smul 𝕜 β] {f : α 𝕜} (hf : measure_theory.ae_strongly_measurable f μ) (c : β) :

Big operators: and #

theorem list.ae_strongly_measurable_prod {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [monoid M] [topological_space M] [has_continuous_mul M] (l : list M)) (hl : (f : α M), f l measure_theory.ae_strongly_measurable f μ) :
measure_theory.ae_strongly_measurable (λ (x : α), (list.map (λ (f : α M), f x) l).prod) μ
theorem list.ae_strongly_measurable_sum {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [add_monoid M] [topological_space M] [has_continuous_add M] (l : list M)) (hl : (f : α M), f l measure_theory.ae_strongly_measurable f μ) :
measure_theory.ae_strongly_measurable (λ (x : α), (list.map (λ (f : α M), f x) l).sum) μ
theorem multiset.ae_strongly_measurable_prod {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [comm_monoid M] [topological_space M] [has_continuous_mul M] (s : multiset M)) (hs : (f : α M), f s measure_theory.ae_strongly_measurable f μ) :
measure_theory.ae_strongly_measurable (λ (x : α), (multiset.map (λ (f : α M), f x) s).prod) μ
theorem multiset.ae_strongly_measurable_sum {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [add_comm_monoid M] [topological_space M] [has_continuous_add M] (s : multiset M)) (hs : (f : α M), f s measure_theory.ae_strongly_measurable f μ) :
measure_theory.ae_strongly_measurable (λ (x : α), (multiset.map (λ (f : α M), f x) s).sum) μ
theorem finset.ae_strongly_measurable_prod' {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [comm_monoid M] [topological_space M] [has_continuous_mul M] {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.ae_strongly_measurable (f i) μ) :
theorem finset.ae_strongly_measurable_sum' {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [add_comm_monoid M] [topological_space M] [has_continuous_add M] {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.ae_strongly_measurable (f i) μ) :
measure_theory.ae_strongly_measurable (s.sum (λ (i : ι), f i)) μ
theorem finset.ae_strongly_measurable_sum {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [add_comm_monoid M] [topological_space M] [has_continuous_add M] {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.ae_strongly_measurable (f i) μ) :
measure_theory.ae_strongly_measurable (λ (a : α), s.sum (λ (i : ι), f i a)) μ
theorem finset.ae_strongly_measurable_prod {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {M : Type u_5} [comm_monoid M] [topological_space M] [has_continuous_mul M] {ι : Type u_2} {f : ι α M} (s : finset ι) (hf : (i : ι), i s measure_theory.ae_strongly_measurable (f i) μ) :
measure_theory.ae_strongly_measurable (λ (a : α), s.prod (λ (i : ι), f i a)) μ

In a space with second countable topology, measurable implies strongly measurable.

In a space with second countable topology, strongly measurable and measurable are equivalent.

@[protected]
@[protected]

A function is almost everywhere strongly measurable if and only if it is almost everywhere measurable, and up to a zero measure set its range is contained in a separable set.

theorem ae_strongly_measurable_of_tendsto_ae {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {ι : Type u_3} [topological_space.pseudo_metrizable_space β] (u : filter ι) [u.ne_bot] [u.is_countably_generated] {f : ι α β} {g : α β} (hf : (i : ι), measure_theory.ae_strongly_measurable (f i) μ) (lim : ∀ᵐ (x : α) μ, filter.tendsto (λ (n : ι), f n x) u (nhds (g x))) :

An almost everywhere sequential limit of almost everywhere strongly measurable functions is almost everywhere strongly measurable.

theorem exists_strongly_measurable_limit_of_tendsto_ae {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] [topological_space.pseudo_metrizable_space β] {f : α β} (hf : (n : ), measure_theory.ae_strongly_measurable (f n) μ) (h_ae_tendsto : ∀ᵐ (x : α) μ, (l : β), filter.tendsto (λ (n : ), f n x) filter.at_top (nhds l)) :
(f_lim : α β) (hf_lim_meas : measure_theory.strongly_measurable f_lim), ∀ᵐ (x : α) μ, filter.tendsto (λ (n : ), f n x) filter.at_top (nhds (f_lim x))

If a sequence of almost everywhere strongly measurable functions converges almost everywhere, one can select a strongly measurable function as the almost everywhere limit.

@[protected]
@[simp]
theorem ae_strongly_measurable_smul_const_iff {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {𝕜 : Type u_5} [nontrivially_normed_field 𝕜] [complete_space 𝕜] {E : Type u_6} [normed_add_comm_group E] [normed_space 𝕜 E] {f : α 𝕜} {c : E} (hc : c 0) :
theorem ae_strongly_measurable_const_smul_iff₀ {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] {f : α β} {G₀ : Type u_7} [group_with_zero G₀] [mul_action G₀ β] [has_continuous_const_smul G₀ β] {c : G₀} (hc : c 0) :
theorem strongly_measurable.apply_continuous_linear_map {α : Type u_1} {𝕜 : Type u_5} [nontrivially_normed_field 𝕜] {E : Type u_6} [normed_add_comm_group E] [normed_space 𝕜 E] {F : Type u_7} [normed_add_comm_group F] [normed_space 𝕜 F] {m : measurable_space α} {φ : α (F →L[𝕜] E)} (hφ : measure_theory.strongly_measurable φ) (v : F) :
theorem continuous_linear_map.ae_strongly_measurable_comp₂ {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {𝕜 : Type u_5} [nontrivially_normed_field 𝕜] {E : Type u_6} [normed_add_comm_group E] [normed_space 𝕜 E] {F : Type u_7} [normed_add_comm_group F] [normed_space 𝕜 F] {G : Type u_8} [normed_add_comm_group G] [normed_space 𝕜 G] (L : E →L[𝕜] F →L[𝕜] G) {f : α E} {g : α F} (hf : measure_theory.ae_strongly_measurable f μ) (hg : measure_theory.ae_strongly_measurable g μ) :
measure_theory.ae_strongly_measurable (λ (x : α), (L (f x)) (g x)) μ

Almost everywhere finitely strongly measurable functions #

@[protected]
noncomputable def measure_theory.ae_fin_strongly_measurable.mk {α : Type u_1} {β : Type u_2} {m : measurable_space α} {μ : measure_theory.measure α} [topological_space β] [has_zero β] (f : α β) (hf : measure_theory.ae_fin_strongly_measurable f μ) :
α β

A fin_strongly_measurable function such that f =ᵐ[μ] hf.mk f. See lemmas fin_strongly_measurable_mk and ae_eq_mk.

Equations

A measurable set t such that f =ᵐ[μ.restrict tᶜ] 0 and sigma_finite (μ.restrict t).

Equations

In a space with second countable topology and a sigma-finite measure, fin_strongly_measurable and measurable are equivalent.

In a space with second countable topology and a sigma-finite measure, ae_fin_strongly_measurable and ae_measurable are equivalent.