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_smul {α : Type u_1} {β : Type u_2} {mα : MeasurableSpace α} {mβ : MeasurableSpace β} (κ : (ProbabilityTheory.kernel α β)) (μ : MeasureTheory.Measure α) (r : ENNReal) :

Invariant measures of kernels #

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

Equations
Instances For