Disintegration of measures on product spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Let ρ
be a finite measure on α × Ω
, where Ω
is a standard Borel space. In mathlib terms, Ω
verifies [nonempty Ω] [topological_space Ω] [polish_space Ω] [measurable_space Ω] [borel_space Ω]
.
Then there exists a kernel ρ.cond_kernel : kernel α Ω
such that for any measurable set
s : set (α × Ω)
, ρ s = ∫⁻ a, ρ.cond_kernel a {x | (a, x) ∈ s} ∂ρ.fst
.
In terms of kernels, ρ.cond_kernel
is such that for any measurable space γ
, we
have a disintegration of the constant kernel from γ
with value ρ
:
kernel.const γ ρ = (kernel.const γ ρ.fst) ⊗ₖ (kernel.prod_mk_left γ (cond_kernel ρ))
,
where ρ.fst
is the marginal measure of ρ
on α
. In particular,
ρ = ((kernel.const unit ρ.fst) ⊗ₖ (kernel.prod_mk_left unit (cond_kernel ρ))) ()
.
In order to obtain a disintegration for any standard Borel space, we use that these spaces embed
measurably into ℝ
: it then suffices to define a suitable kernel for Ω = ℝ
. In the real case,
we define a conditional kernel by taking for each a : α
the measure associated to the Stieltjes
function cond_cdf ρ a
(the conditional cumulative distribution function).
Main definitions #
measure_theory.measure.cond_kernel ρ : kernel α Ω
: conditional kernel described above.
Main statements #
probability_theory.lintegral_cond_kernel
:∫⁻ a, ∫⁻ ω, f (a, ω) ∂(ρ.cond_kernel a) ∂ρ.fst = ∫⁻ x, f x ∂ρ
probability_theory.lintegral_cond_kernel_mem
:∫⁻ a, ρ.cond_kernel a {x | (a, x) ∈ s} ∂ρ.fst = ρ s
probability_theory.kernel.const_eq_comp_prod
:kernel.const γ ρ = (kernel.const γ ρ.fst) ⊗ₖ (kernel.prod_mk_left γ ρ.cond_kernel)
probability_theory.measure_eq_comp_prod
:ρ = ((kernel.const unit ρ.fst) ⊗ₖ (kernel.prod_mk_left unit ρ.cond_kernel)) ()
Disintegration of measures on α × ℝ
#
Conditional measure on the second space of the product given the value on the first, as a
kernel. Use the more general cond_kernel
.
Equations
- probability_theory.cond_kernel_real ρ = ⟨λ (a : α), (probability_theory.cond_cdf ρ a).measure, _⟩
Instances for probability_theory.cond_kernel_real
Disintegration of measures on Polish Borel spaces #
Since every standard Borel space embeds measurably into ℝ
, we can generalize the disintegration
property on ℝ
to all these spaces.
Existence of a conditional kernel. Use the definition cond_kernel
to get that kernel.
Conditional kernel of a measure on a product space: a Markov kernel such that
ρ = ((kernel.const unit ρ.fst) ⊗ₖ (kernel.prod_mk_left unit ρ.cond_kernel)) ()
(see probability_theory.measure_eq_comp_prod
).
Equations
- ρ.cond_kernel = _.some
Instances for measure_theory.measure.cond_kernel
Disintegration of finite product measures on α × Ω
, where Ω
is Polish Borel. Such a
measure can be written as the composition-product of the constant kernel with value ρ.fst
(marginal measure over α
) and a Markov kernel from α
to Ω
. We call that Markov kernel
probability_theory.cond_kernel ρ
.
Disintegration of constant kernels. A constant kernel on a product space α × Ω
, where Ω
is Polish Borel, can be written as the composition-product of the constant kernel with value ρ.fst
(marginal measure over α
) and a Markov kernel from α
to Ω
. We call that Markov kernel
probability_theory.cond_kernel ρ
.
Integrability #
We place these lemmas in the measure_theory
namespace to enable dot notation.