mathlib3 documentation

probability.kernel.condexp

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 #

Main statements #

theorem probability_theory.measurable_id'' {Ω : Type u_1} {m mΩ : measurable_space Ω} (hm : m mΩ) :
theorem probability_theory.ae_measurable_id'' {Ω : Type u_1} {m mΩ : measurable_space Ω} (μ : measure_theory.measure Ω) (hm : m mΩ) :
theorem measure_theory.ae_strongly_measurable.comp_snd_map_prod_id {Ω : Type u_1} {F : Type u_2} {m mΩ : measurable_space Ω} {μ : measure_theory.measure Ω} {f : Ω F} [topological_space F] (hm : m mΩ) (hf : measure_theory.ae_strongly_measurable f μ) :
measure_theory.ae_strongly_measurable (λ (x : Ω × Ω), f x.snd) (measure_theory.measure.map (λ (ω : Ω), (id ω, id ω)) μ)
theorem measure_theory.integrable.comp_snd_map_prod_id {Ω : Type u_1} {F : Type u_2} {m mΩ : measurable_space Ω} {μ : measure_theory.measure Ω} {f : Ω F} [normed_add_comm_group F] (hm : m mΩ) (hf : measure_theory.integrable f μ) :
measure_theory.integrable (λ (x : Ω × Ω), f x.snd) (measure_theory.measure.map (λ (ω : Ω), (id ω, id ω)) μ)
@[irreducible]

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 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 ω).