Documentation

Mathlib.Probability.Kernel.Invariance

Invariance of measures along a kernel #

We say that a measure μ is invariant with respect to a kernel κ if its push-forward along the kernel μ.bind κ is the same measure.

Main definitions #

Useful lemmas #

Push-forward of measures along a kernel #

@[simp]
theorem ProbabilityTheory.kernel.bind_add {α : Type u_1} {β : Type u_2} {mα : MeasurableSpace α} {mβ : MeasurableSpace β} (μ : MeasureTheory.Measure α) (ν : MeasureTheory.Measure α) (κ : (ProbabilityTheory.kernel α β)) :
(μ + ν).bind κ = μ.bind κ + ν.bind κ
@[simp]
theorem ProbabilityTheory.kernel.bind_smul {α : Type u_1} {β : Type u_2} {mα : MeasurableSpace α} {mβ : MeasurableSpace β} (κ : (ProbabilityTheory.kernel α β)) (μ : MeasureTheory.Measure α) (r : ENNReal) :
(r μ).bind κ = r μ.bind κ

Invariant measures of kernels #

A measure μ is invariant with respect to the kernel κ if the push-forward measure of μ along κ equals μ.

Equations
Instances For
    theorem ProbabilityTheory.kernel.Invariant.def {α : Type u_1} {mα : MeasurableSpace α} {κ : (ProbabilityTheory.kernel α α)} {μ : MeasureTheory.Measure α} (hκ : ProbabilityTheory.kernel.Invariant κ μ) :
    μ.bind κ = μ