Conditional expectation in L2 #
This file contains one step of the construction of the conditional expectation, which is completed
in MeasureTheory.Function.ConditionalExpectation.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 #
condExpL2
: Conditional expectation of a function in L2 with respect to a sigma-algebra: it is the orthogonal projection on the subspacelpMeas
.
Implementation notes #
Most of the results in this file are valid for a complete real normed space F
.
However, some lemmas also use 𝕜 : RCLike
:
condExpL2
is defined only for anInnerProductSpace
for now, and we use𝕜
for its field.- results about scalar multiplication are stated not only for
ℝ
but also for𝕜
if we happen to haveNormedSpace 𝕜 F
.
Conditional expectation of a function in L2 with respect to a sigma-algebra
Equations
- MeasureTheory.condExpL2 E 𝕜 hm = orthogonalProjection (MeasureTheory.lpMeas E 𝕜 m 2 μ)
Instances For
Alias of MeasureTheory.condExpL2
.
Conditional expectation of a function in L2 with respect to a sigma-algebra
Equations
Instances For
Alias of MeasureTheory.integrableOn_condExpL2_of_measure_ne_top
.
Alias of MeasureTheory.integrable_condExpL2_of_isFiniteMeasure
.
Alias of MeasureTheory.norm_condExpL2_le_one
.
Alias of MeasureTheory.norm_condExpL2_le
.
Alias of MeasureTheory.eLpNorm_condExpL2_le
.
Alias of MeasureTheory.norm_condExpL2_coe_le
.
Alias of MeasureTheory.integral_condExpL2_eq_of_fin_meas_real
.
Alias of MeasureTheory.lintegral_nnnorm_condExpL2_indicator_le_real
.
condExpL2
commutes with taking inner products with constants. See the lemma
condExpL2_comp_continuousLinearMap
for a more general result about commuting with continuous
linear maps.
Alias of MeasureTheory.condExpL2_const_inner
.
condExpL2
commutes with taking inner products with constants. See the lemma
condExpL2_comp_continuousLinearMap
for a more general result about commuting with continuous
linear maps.
condExpL2
verifies the equality of integrals defining the conditional expectation.
Alias of MeasureTheory.integral_condExpL2_eq
.
condExpL2
verifies the equality of integrals defining the conditional expectation.
Alias of MeasureTheory.condExpL2_indicator_eq_toSpanSingleton_comp
.
Alias of MeasureTheory.setLIntegral_nnnorm_condExpL2_indicator_le
.
Alias of MeasureTheory.lintegral_nnnorm_condExpL2_indicator_le
.
If the measure μ.trim hm
is sigma-finite, then the conditional expectation of a measurable set
with finite measure is integrable.
Alias of MeasureTheory.integrable_condExpL2_indicator
.
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
- One or more equations did not get rendered due to their size.
Instances For
Alias of MeasureTheory.condExpIndSMul
.
Conditional expectation of the indicator of a measurable set with finite measure, in L2.
Instances For
Alias of MeasureTheory.condExpIndSMul_add
.
Alias of MeasureTheory.condExpIndSMul_smul
.
Alias of MeasureTheory.condExpIndSMul_smul'
.
Alias of MeasureTheory.condExpIndSMul_ae_eq_smul
.
Alias of MeasureTheory.setLIntegral_nnnorm_condExpIndSMul_le
.
If the measure μ.trim hm
is sigma-finite, then the conditional expectation of a measurable set
with finite measure is integrable.
Alias of MeasureTheory.integrable_condExpIndSMul
.
If the measure μ.trim hm
is sigma-finite, then the conditional expectation of a measurable set
with finite measure is integrable.
Alias of MeasureTheory.condExpIndSMul_empty
.
Alias of MeasureTheory.setIntegral_condExpIndSMul
.
Alias of MeasureTheory.condExpL2_indicator_nonneg
.
Alias of MeasureTheory.condExpIndSMul_nonneg
.