Documentation

Mathlib.Probability.Kernel.RadonNikodym

Radon-Nikodym derivative and Lebesgue decomposition for kernels #

Let γ be a countably generated measurable space and κ, η : kernel α γ be finite kernels. Then there exists a function kernel.rnDeriv κ η : α → γ → ℝ≥0∞ jointly measurable on α × γ and a kernel kernel.singularPart κ η : kernel α γ such that

Furthermore, the sets {a | κ a ≪ η a} and {a | κ a ⟂ₘ η a} are measurable.

The construction of the derivative starts from kernel.density: for two finite kernels κ' : kernel α (γ × β) and η' : kernel α γ with fst κ' ≤ η', the function density κ' η' : α → γ → Set β → ℝ is jointly measurable in the first two arguments and satisfies that for all a : α and all measurable sets s : Set β and A : Set γ, ∫ x in A, density κ' η' a x s ∂(η' a) = (κ' a (A ×ˢ s)).toReal. We use that definition for β = Unit and κ' = map κ (fun a ↦ (a, ())). We can't choose η' = η in general because we might not have κ ≤ η, but if we could, we would get a measurable function f with the property κ = withDensity η f, which is the decomposition we want for κ ≤ η. To circumvent that difficulty, we take η' = κ + η and thus define rnDerivAux κ η. Finally, rnDeriv κ η a x is given by ENNReal.ofReal (rnDerivAux κ (κ + η) a x) / ENNReal.ofReal (1 - rnDerivAux κ (κ + η) a x). Up to some conversions between and ℝ≥0, the singular part is withDensity (κ + η) (rnDerivAux κ (κ + η) - (1 - rnDerivAux κ (κ + η)) * rnDeriv κ η).

The countably generated measurable space assumption is not needed to have a decomposition for measures, but the additional difficulty with kernels is to obtain joint measurability of the derivative. This is why we can't simply define rnDeriv κ η by a ↦ (κ a).rnDeriv (ν a) everywhere (although rnDeriv κ η has that value almost everywhere). See the construction of kernel.density for details on how the countably generated hypothesis is used.

Main definitions #

Main statements #

References #

Theorem 1.28 in [O. Kallenberg, Random Measures, Theory and Applications][kallenberg2017].

TODO #

noncomputable def ProbabilityTheory.kernel.rnDerivAux {α : Type u_1} {γ : Type u_2} {mα : MeasurableSpace α} {mγ : MeasurableSpace γ} [MeasurableSpace.CountablyGenerated γ] (κ : (ProbabilityTheory.kernel α γ)) (η : (ProbabilityTheory.kernel α γ)) (a : α) (x : γ) :

Auxiliary function used to define ProbabilityTheory.kernel.rnDeriv and ProbabilityTheory.kernel.singularPart.

This has the properties we want for a Radon-Nikodym derivative only if κ ≪ ν. The definition of rnDeriv κ η will be built from rnDerivAux κ (κ + η).

Equations
Instances For
    theorem ProbabilityTheory.kernel.rnDerivAux_nonneg {α : Type u_1} {γ : Type u_2} {mα : MeasurableSpace α} {mγ : MeasurableSpace γ} [MeasurableSpace.CountablyGenerated γ] {κ : (ProbabilityTheory.kernel α γ)} {η : (ProbabilityTheory.kernel α γ)} (hκη : κ η) {a : α} {x : γ} :
    theorem ProbabilityTheory.kernel.rnDerivAux_le_one {α : Type u_1} {γ : Type u_2} {mα : MeasurableSpace α} {mγ : MeasurableSpace γ} [MeasurableSpace.CountablyGenerated γ] {κ : (ProbabilityTheory.kernel α γ)} {η : (ProbabilityTheory.kernel α γ)} (hκη : κ η) {a : α} {x : γ} :
    theorem ProbabilityTheory.kernel.set_lintegral_rnDerivAux {α : Type u_1} {γ : Type u_2} {mα : MeasurableSpace α} {mγ : MeasurableSpace γ} [MeasurableSpace.CountablyGenerated γ] (κ : (ProbabilityTheory.kernel α γ)) (η : (ProbabilityTheory.kernel α γ)) [ProbabilityTheory.IsFiniteKernel κ] [ProbabilityTheory.IsFiniteKernel η] (a : α) {s : Set γ} (hs : MeasurableSet s) :
    ∫⁻ (x : γ) in s, ENNReal.ofReal (ProbabilityTheory.kernel.rnDerivAux κ (κ + η) a x)(κ + η) a = (κ a) s

    A set of points in α × γ related to the absolute continuity / mutual singularity of κ and η.

    Equations
    Instances For

      A set of points in α × γ related to the absolute continuity / mutual singularity of κ and η. That is,

      • withDensity η (rnDeriv κ η) a (mutuallySingularSetSlice κ η a) = 0,
      • singularPart κ η a (mutuallySingularSetSlice κ η a)ᶜ = 0.
      Equations
      Instances For
        @[irreducible]
        noncomputable def ProbabilityTheory.kernel.rnDeriv {α : Type u_3} {γ : Type u_4} {mα : MeasurableSpace α} {mγ : MeasurableSpace γ} [MeasurableSpace.CountablyGenerated γ] (κ : (ProbabilityTheory.kernel α γ)) (η : (ProbabilityTheory.kernel α γ)) (a : α) (x : γ) :

        Radon-Nikodym derivative of the kernel κ with respect to the kernel η.

        Equations
        Instances For
          @[irreducible]

          Singular part of the kernel κ with respect to the kernel η.

          Equations
          Instances For

            The singular part of κ with respect to η is mutually singular with η.

            Lebesgue decomposition of a finite kernel κ with respect to another one η. κ is the sum of an abolutely continuous part withDensity η (rnDeriv κ η) and a singular part singularPart κ η.

            The set of points a : α such that κ a ≪ η a is measurable.

            The set of points a : α such that κ a ⟂ₘ η a is measurable.