Conditional expectation in L2 #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains one step of the construction of the conditional expectation, which is completed
in measure_theory.function.conditional_expectation.basic
. See that file for a description of the
full process.
We build the conditional expectation of an L²
function, as an element of L²
. This is the
orthogonal projection on the subspace of almost everywhere m
-measurable functions.
Main definitions #
condexp_L2
: Conditional expectation of a function in L2 with respect to a sigma-algebra: it is the orthogonal projection on the subspaceLp_meas
.
Implementation notes #
Most of the results in this file are valid for a complete real normed space F
.
However, some lemmas also use 𝕜 : is_R_or_C
:
condexp_L2
is defined only for aninner_product_space
for now, and we use𝕜
for its field.- results about scalar multiplication are stated not only for
ℝ
but also for𝕜
if we happen to havenormed_space 𝕜 F
.
Conditional expectation of a function in L2 with respect to a sigma-algebra
Equations
- measure_theory.condexp_L2 𝕜 hm = orthogonal_projection (measure_theory.Lp_meas E 𝕜 m 2 μ)
condexp_L2
commutes with taking inner products with constants. See the lemma
condexp_L2_comp_continuous_linear_map
for a more general result about commuting with continuous
linear maps.
condexp_L2
verifies the equality of integrals defining the conditional expectation.
If the measure μ.trim hm
is sigma-finite, then the conditional expectation of a measurable set
with finite measure is integrable.
Conditional expectation of the indicator of a measurable set with finite measure, in L2.
Equations
- measure_theory.condexp_ind_smul hm hs hμs x = ⇑(continuous_linear_map.comp_LpL 2 μ (continuous_linear_map.to_span_singleton ℝ x)) ↑(⇑(measure_theory.condexp_L2 ℝ hm) (measure_theory.indicator_const_Lp 2 hs hμs 1))
If the measure μ.trim hm
is sigma-finite, then the conditional expectation of a measurable set
with finite measure is integrable.