Conditional expectation #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We build the conditional expectation of an integrable function f with value in a Banach space
with respect to a measure μ (defined on a measurable space structure m0) and a measurable space
structure m with hm : m ≤ m0 (a sub-sigma-algebra). This is an m-strongly measurable
function μ[f|hm] which is integrable and verifies ∫ x in s, μ[f|hm] x ∂μ = ∫ x in s, f x ∂μ
for all m-measurable sets s. It is unique as an element of L¹.
The construction is done in four steps:
- Define the conditional expectation of an
L²function, as an element ofL². This is the orthogonal projection on the subspace of almost everywherem-measurable functions. - Show that the conditional expectation of the indicator of a measurable set with finite measure
is integrable and define a map
set α → (E →L[ℝ] (α →₁[μ] E))which to a set associates a linear map. That linear map sendsx ∈ Eto the conditional expectation of the indicator of the set with valuex. - Extend that map to
condexp_L1_clm : (α →₁[μ] E) →L[ℝ] (α →₁[μ] E). This is done using the same construction as the Bochner integral (see the filemeasure_theory/integral/set_to_L1). - Define the conditional expectation of a function
f : α → E, which is an integrable functionα → Eequal to 0 iffis not integrable, and equal to anm-measurable representative ofcondexp_L1_clmapplied to[f], the equivalence class offinL¹.
The first step is done in measure_theory.function.conditional_expectation.condexp_L2, the two
next steps in measure_theory.function.conditional_expectation.condexp_L1 and the final step is
performed in this file.
Main results #
The conditional expectation and its properties
condexp (m : measurable_space α) (μ : measure α) (f : α → E): conditional expectation offwith respect tom.integrable_condexp:condexpis integrable.strongly_measurable_condexp:condexpism-strongly-measurable.set_integral_condexp (hf : integrable f μ) (hs : measurable_set[m] s): ifm ≤ m0(the σ-algebra over which the measure is defined), then the conditional expectation verifies∫ x in s, condexp m μ f x ∂μ = ∫ x in s, f x ∂μfor anym-measurable sets.
While condexp is function-valued, we also define condexp_L1 with value in L1 and a continuous
linear map condexp_L1_clm from L1 to L1. condexp should be used in most cases.
Uniqueness of the conditional expectation
ae_eq_condexp_of_forall_set_integral_eq: an a.e.m-measurable function which verifies the equality of integrals is a.e. equal tocondexp.
Notations #
For a measure μ defined on a measurable space structure m0, another measurable space structure
m with hm : m ≤ m0 (a sub-σ-algebra) and a function f, we define the notation
μ[f|m] = condexp m μ f.
Tags #
conditional expectation, conditional expected value
Conditional expectation of a function. It is defined as 0 if any one of the following conditions is true:
mis not a sub-σ-algebra ofm0,μis not σ-finite with respect tom,fis not integrable.
Equations
- measure_theory.condexp m μ f = dite (m ≤ m0) (λ (hm : m ≤ m0), dite (measure_theory.sigma_finite (μ.trim hm) ∧ measure_theory.integrable f μ) (λ (h : measure_theory.sigma_finite (μ.trim hm) ∧ measure_theory.integrable f μ), ite (measure_theory.strongly_measurable f) f (measure_theory.ae_strongly_measurable'.mk ⇑(measure_theory.condexp_L1 hm μ f) _)) (λ (h : ¬(measure_theory.sigma_finite (μ.trim hm) ∧ measure_theory.integrable f μ)), 0)) (λ (hm : ¬m ≤ m0), 0)
The integral of the conditional expectation μ[f|hm] over an m-measurable set is equal to
the integral of f on that set.
Uniqueness of the conditional expectation
If a function is a.e. m-measurable, verifies an integrability condition and has same integral
as f on all m-measurable sets, then it is a.e. equal to μ[f|hm].
Lebesgue dominated convergence theorem: sufficient conditions under which almost
everywhere convergence of a sequence of functions implies the convergence of their image by
condexp_L1.
If two sequences of functions have a.e. equal conditional expectations at each step, converge and verify dominated convergence hypotheses, then the conditional expectations of their limits are a.e. equal.