Conditional expectation #
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 condexpL1CLM : (α →₁[μ] E) →L[ℝ] (α →₁[μ] E). This is done using the same construction as the Bochner integral (see the fileMeasureTheory/Integral/SetToL1).
- 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 ofcondexpL1CLMapplied to[f], the equivalence class offinL¹.
The first step is done in MeasureTheory.Function.ConditionalExpectation.CondexpL2, the two
next steps in MeasureTheory.Function.ConditionalExpectation.CondexpL1 and the final step is
performed in this file.
Main results #
The conditional expectation and its properties
- condexp (m : MeasurableSpace α) (μ : Measure α) (f : α → E): conditional expectation of- fwith respect to- m.
- integrable_condexp:- condexpis integrable.
- stronglyMeasurable_condexp:- condexpis- m-strongly-measurable.
- setIntegral_condexp (hf : Integrable f μ) (hs : MeasurableSet[m] s): if- m ≤ 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 any- m-measurable set- s.
While condexp is function-valued, we also define condexpL1 with value in L1 and a continuous
linear map condexpL1CLM from L1 to L1. condexp should be used in most cases.
Uniqueness of the conditional expectation
- ae_eq_condexp_of_forall_setIntegral_eq: an a.e.- m-measurable function which verifies the equality of integrals is a.e. equal to- condexp.
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 of- m0,
- μis not σ-finite with respect to- m,
- fis not integrable.
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
The integral of the conditional expectation μ[f|hm] over an m-measurable set is equal to
the integral of f on that set.
Alias of MeasureTheory.setIntegral_condexp.
The integral of the conditional expectation μ[f|hm] over an m-measurable set is equal to
the integral of f on that set.
Total probability law using condexp as conditional probability.
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].
Alias of MeasureTheory.ae_eq_condexp_of_forall_setIntegral_eq.
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
condexpL1.
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.