Proper kernels #
This file defines properness of measure kernels.
For two σ-algebras 𝓑 ≤ 𝓧
, a 𝓑, 𝓧
-kernel π : X → Measure X
is proper if
∫ x, g x * f x ∂(π x₀) = g x₀ * ∫ x, f x ∂(π x₀)
for all x₀ : X
, 𝓧
-measurable function f
and 𝓑
-measurable function g
.
By the standard machine, this is equivalent to having that, for all B ∈ 𝓑
, π
restricted to B
is the same as π
times the indicator of B
.
This should be thought of as the condition under which one can meaningfully restrict a kernel to an event.
TODO #
Prove the integral
versions of the lintegral
lemmas below
For two σ-algebras 𝓑 ≤ 𝓧
on a space X
, a 𝓑, 𝓧
-kernel π : X → Measure X
is proper if
∫ x, g x * f x ∂(π x₀) = g x₀ * ∫ x, f x ∂(π x₀)
for all x₀ : X
, 𝓧
-measurable function f
and 𝓑
-measurable function g
.
By the standard machine, this is equivalent to having that, for all B ∈ 𝓑
, π
restricted to B
is the same as π
times the indicator of B
.
To avoid assuming 𝓑 ≤ 𝓧
in the definition, we replace 𝓑
by 𝓑 ⊓ 𝓧
in the restriction.
- restrict_eq_indicator_smul' ⦃B : Set X⦄ (hB : MeasurableSet B) (x : X) : (π.restrict ⋯) x = B.indicator (fun (x : X) => 1) x • π x
Instances For
Alias of the forward direction of ProbabilityTheory.Kernel.isProper_iff_restrict_eq_indicator_smul
.
Alias of the reverse direction of ProbabilityTheory.Kernel.isProper_iff_restrict_eq_indicator_smul
.
Alias of the forward direction of ProbabilityTheory.Kernel.isProper_iff_inter_eq_indicator_mul
.
Alias of the reverse direction of ProbabilityTheory.Kernel.isProper_iff_inter_eq_indicator_mul
.