With Density #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
For an s-finite kernel κ : kernel α β
and a function f : α → β → ℝ≥0∞
which is finite
everywhere, we define with_density κ f
as the kernel a ↦ (κ a).with_density (f a)
. This is
an s-finite kernel.
Main definitions #
probability_theory.kernel.with_density κ (f : α → β → ℝ≥0∞)
: kernela ↦ (κ a).with_density (f a)
. It is defined ifκ
is s-finite. Iff
is finite everywhere, then this is also an s-finite kernel. The class of s-finite kernels is the smallest class of kernels that contains finite kernels and which is stable bywith_density
. Integral:∫⁻ b, g b ∂(with_density κ f a) = ∫⁻ b, f a b * g b ∂(κ a)
Main statements #
probability_theory.kernel.lintegral_with_density
:∫⁻ b, g b ∂(with_density κ f a) = ∫⁻ b, f a b * g b ∂(κ a)
Kernel with image (κ a).with_density (f a)
if function.uncurry f
is measurable, and
with image 0 otherwise. If function.uncurry f
is measurable, it satisfies
∫⁻ b, g b ∂(with_density κ f hf a) = ∫⁻ b, f a b * g b ∂(κ a)
.
Equations
- probability_theory.kernel.with_density κ f = dite (measurable (function.uncurry f)) (λ (hf : measurable (function.uncurry f)), ⟨λ (a : α), (⇑κ a).with_density (f a), _⟩) (λ (hf : ¬measurable (function.uncurry f)), 0)
Instances for probability_theory.kernel.with_density
If a kernel κ
is finite and a function f : α → β → ℝ≥0∞
is bounded, then with_density κ f
is finite.
Auxiliary lemma for is_s_finite_kernel_with_density
.
If a kernel κ
is finite, then with_density κ f
is s-finite.
For a s-finite kernel κ
and a function f : α → β → ℝ≥0∞
which is everywhere finite,
with_density κ f
is s-finite.
For a s-finite kernel κ
and a function f : α → β → ℝ≥0
, with_density κ f
is s-finite.