Kernel associated with a conditional expectation #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define condexp_kernel μ m
, a kernel from Ω
to Ω
such that for all integrable functions f
,
μ[f | m] =ᵐ[μ] λ ω, ∫ y, f y ∂(condexp_kernel μ m ω)
.
This kernel is defined if Ω
is a standard Borel space. In general, μ⟦s | m⟧
maps a measurable
set s
to a function Ω → ℝ≥0∞
, and for all s
that map is unique up to a μ
-null set. For all
a
, the map from sets to ℝ≥0∞
that we obtain that way verifies some of the properties of a
measure, but the fact that the μ
-null set depends on s
can prevent us from finding versions of
the conditional expectation that combine into a true measure. The standard Borel space assumption
on Ω
allows us to do so.
Main definitions #
condexp_kernel μ m
: kernel such thatμ[f | m] =ᵐ[μ] λ ω, ∫ y, f y ∂(condexp_kernel μ m ω)
.
Main statements #
condexp_ae_eq_integral_condexp_kernel
:μ[f | m] =ᵐ[μ] λ ω, ∫ y, f y ∂(condexp_kernel μ m ω)
.
Kernel associated with the conditional expectation with respect to a σ-algebra. It satisfies
μ[f | m] =ᵐ[μ] λ ω, ∫ y, f y ∂(condexp_kernel μ m ω)
.
It is defined as the conditional distribution of the identity given the identity, where the second
identity is understood as a map from Ω
with the σ-algebra mΩ
to Ω
with σ-algebra m
.
Equations
The conditional expectation of f
with respect to a σ-algebra m
is almost everywhere equal to
the integral ∫ y, f y ∂(condexp_kernel μ m ω)
.