Strongly measurable and finitely strongly measurable functions #
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.
If the target space has a second countable topology, strongly measurable and measurable are equivalent.
Functions in Lp for 0 < p < ∞ are finitely strongly measurable.
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 #
-
strongly_measurable f:f : α → βis the limit of a sequencefs : ℕ → simple_func α β. -
fin_strongly_measurable f μ:f : α → βis the limit of a sequencefs : ℕ → simple_func α βsuch that for alln ∈ ℕ, the measure of the support offs nis finite. -
ae_fin_strongly_measurable f μ:fis almost everywhere equal to afin_strongly_measurablefunction. -
ae_fin_strongly_measurable.sigma_finite_set: a measurable settsuch thatf =ᵐ[μ.restrict tᶜ] 0andμ.restrict tis sigma-finite.
Main statements #
ae_fin_strongly_measurable.exists_set_sigma_finite: there exists a measurable settsuch thatf =ᵐ[μ.restrict tᶜ] 0andμ.restrict tis sigma-finite.mem_ℒp.ae_fin_strongly_measurable: ifmem_ℒp f p μwith0 < p < ∞, thenae_fin_strongly_measurable f μ.Lp.fin_strongly_measurable: for0 < p < ∞,Lpfunctions are finitely strongly measurable.
References #
- Hytönen, Tuomas, Jan Van Neerven, Mark Veraar, and Lutz Weis. Analysis in Banach spaces. Springer, 2016.
A function is strongly_measurable if it is the limit of simple functions.
Equations
- measure_theory.strongly_measurable f = ∃ (fs : ℕ → measure_theory.simple_func α β), ∀ (x : α), filter.tendsto (λ (n : ℕ), ⇑(fs n) x) filter.at_top (𝓝 (f x))
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
- measure_theory.fin_strongly_measurable f μ = ∃ (fs : ℕ → measure_theory.simple_func α β), (∀ (n : ℕ), ⇑μ (function.support ⇑(fs n)) < ⊤) ∧ ∀ (x : α), filter.tendsto (λ (n : ℕ), ⇑(fs n) x) filter.at_top (𝓝 (f x))
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
- measure_theory.ae_fin_strongly_measurable f μ = ∃ (g : α → β), measure_theory.fin_strongly_measurable g μ ∧ f =ᵐ[μ] g
Strongly measurable functions #
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
- hf.approx = Exists.some hf
If the measure is sigma-finite, all strongly measurable functions are
fin_strongly_measurable.
A strongly measurable function is measurable.
In a space with second countable topology, measurable implies strongly measurable.
In a space with second countable topology, strongly measurable and measurable are equivalent.
Finitely strongly measurable functions #
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
- hf.approx = Exists.some hf
A finitely strongly measurable function is measurable.
A measurable set t such that f =ᵐ[μ.restrict tᶜ] 0 and sigma_finite (μ.restrict t).
Equations
- hf.sigma_finite_set = _.some
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.