Documentation

Mathlib.Probability.Kernel.Disintegration.Basic

Disintegration of kernels and measures #

Let κ : kernel α (β × Ω) be a finite kernel, where Ω is a standard Borel space. Then if α is countable or β has a countably generated σ-algebra (for example if it is standard Borel), then there exists a kernel (α × β) Ω called conditional kernel and denoted by condKernel κ such that κ = fst κ ⊗ₖ condKernel κ. We also define a conditional kernel for a measure ρ : Measure (β × Ω), where Ω is a standard Borel space. This is a kernel β Ω denoted by ρ.condKernel such that ρ = ρ.fst ⊗ₘ ρ.condKernel.

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 Ω = ℝ.

For κ : kernel α (β × ℝ), the construction of the conditional kernel proceeds as follows:

The first step (building the measurable function on ) is done differently depending on whether α is countable or not.

The conditional kernel is defined under the typeclass assumption CountableOrCountablyGenerated α β, which encodes the property Countable α ∨ CountablyGenerated β.

Properties of integrals involving condKernel are collated in the file Integral.lean. The conditional kernel is unique (almost everywhere w.r.t. fst κ): this is proved in the file Unique.lean.

Main definitions #

Main statements #

Disintegration of kernels from α to γ × ℝ for countably generated γ #

Taking the kernel density of intervals Iic q for q : ℚ gives a function with the property isRatCondKernelCDF.

The conditional kernel CDF of a kernel κ : kernel α (γ × ℝ), where γ is countably generated.

Equations
  • One or more equations did not get rendered due to their size.
Instances For

    Auxiliary definition for ProbabilityTheory.kernel.condKernel. A conditional kernel for κ : kernel α (γ × ℝ) where γ is countably generated.

    Equations
    Instances For

      Disintegration of kernels on standard Borel spaces #

      Since every standard Borel space embeds measurably into , we can generalize a disintegration property on to all these spaces.

      Auxiliary definition for ProbabilityTheory.kernel.condKernel. A Borel space Ω embeds measurably into (with embedding e), hence we can get a kernel α Ω from a kernel α ℝ by taking the comap by e. Here we take the comap of a modification of η : kernel α ℝ, useful when η a is a probability measure with all its mass on range e almost everywhere with respect to some measure and we want to ensure that the comap is a Markov kernel. We thus take the comap by e of a kernel defined piecewise: η when η a (range (embeddingReal Ω))ᶜ = 0, and an arbitrary deterministic kernel otherwise.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        For κ' := map κ (Prod.map (id : β → β) e) (measurable_id.prod_map he.measurable), the hypothesis is fst κ' ⊗ₖ η = κ'. With that hypothesis, fst κ ⊗ₖ borelMarkovFromReal κ η = κ.

        Auxiliary definition for ProbabilityTheory.kernel.condKernel. A conditional kernel for κ : kernel α (γ × Ω) where γ is countably generated and Ω is standard Borel.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          Auxiliary definition for MeasureTheory.Measure.condKernel and ProbabilityTheory.kernel.condKernel. A conditional kernel for κ : kernel Unit (α × Ω) where Ω is standard Borel.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[irreducible]

            Conditional kernel of a measure on a product space: a Markov kernel such that ρ = ρ.fst ⊗ₘ ρ.condKernel (see MeasureTheory.Measure.compProd_fst_condKernel).

            Equations
            Instances For

              Disintegration of finite product measures on α × Ω, where Ω is standard Borel. Such a measure can be written as the composition-product of ρ.fst (marginal measure over α) and a Markov kernel from α to Ω. We call that Markov kernel ρ.condKernel.

              theorem MeasureTheory.Measure.condKernel_apply_of_ne_zero {α : Type u_1} {Ω : Type u_4} {mα : MeasurableSpace α} [MeasurableSpace Ω] [StandardBorelSpace Ω] [Nonempty Ω] {ρ : MeasureTheory.Measure (α × Ω)} [MeasureTheory.IsFiniteMeasure ρ] [MeasurableSingletonClass α] {x : α} (hx : (MeasureTheory.Measure.fst ρ) {x} 0) (s : Set Ω) :
              ((MeasureTheory.Measure.condKernel ρ) x) s = ((MeasureTheory.Measure.fst ρ) {x})⁻¹ * ρ ({x} ×ˢ s)

              If the singleton {x} has non-zero mass for ρ.fst, then for all s : Set Ω, ρ.condKernel x s = (ρ.fst {x})⁻¹ * ρ ({x} ×ˢ s) .

              noncomputable def ProbabilityTheory.kernel.condKernelCountable {α : Type u_1} {β : Type u_2} {Ω : Type u_4} {mα : MeasurableSpace α} {mβ : MeasurableSpace β} [MeasurableSpace Ω] [StandardBorelSpace Ω] [Nonempty Ω] [Countable α] (κ : (ProbabilityTheory.kernel α (β × Ω))) [ProbabilityTheory.IsFiniteKernel κ] :

              Auxiliary definition for ProbabilityTheory.kernel.condKernel. A conditional kernel for κ : kernel α (β × Ω) where α is countable and Ω is standard Borel.

              Equations
              Instances For
                @[irreducible]

                Conditional kernel of a kernel κ : kernel α (β × Ω): a Markov kernel such that fst κ ⊗ₖ condKernel κ = κ (see MeasureTheory.Measure.compProd_fst_condKernel). It exists whenever Ω is standard Borel and either α is countable or β is countably generated.

                Equations
                Instances For

                  Disintegration of finite kernels. The composition-product of fst κ and condKernel κ is equal to κ.