Conditional cumulative distribution function #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Given ρ : measure (α × ℝ)
, we define the conditional cumulative distribution function
(conditional cdf) of ρ
. It is a function cond_cdf ρ : α → ℝ → ℝ
such that if ρ
is a finite
measure, then for all a : α
cond_cdf ρ a
is monotone and right-continuous with limit 0 at -∞
and limit 1 at +∞, and such that for all x : ℝ
, a ↦ cond_cdf ρ a x
is measurable. For all
x : ℝ
and measurable set s
, that function satisfies
∫⁻ a in s, ennreal.of_real (cond_cdf ρ a x) ∂ρ.fst = ρ (s ×ˢ Iic x)
.
Main definitions #
probability_theory.cond_cdf ρ : α → stieltjes_function
: the conditional cdf ofρ : measure (α × ℝ)
. Astieltjes_function
is a functionℝ → ℝ
which is monotone and right-continuous.
Main statements #
probability_theory.set_lintegral_cond_cdf
: for alla : α
andx : ℝ
, all measurable sets
,∫⁻ a in s, ennreal.of_real (cond_cdf ρ a x) ∂ρ.fst = ρ (s ×ˢ Iic x)
.
References #
The construction of the conditional cdf in this file follows the proof of Theorem 3.4 in O. Kallenberg, Foundations of modern probability.
TODO #
Monotone convergence for an infimum over a directed family and indexed by a countable type
Measure on α
such that for a measurable set s
, ρ.Iic_snd r s = ρ (s ×ˢ Iic r)
.
Auxiliary definitions #
We build towards the definition of probability_theory.cond_cdf
. We first define
probability_theory.pre_cdf
, a function defined on α × ℚ
with the properties of a cdf almost
everywhere. We then introduce probability_theory.cond_cdf_rat
, a function on α × ℚ
which has
the properties of a cdf for all a : α
. We finally extend to ℝ
.
pre_cdf
is the Radon-Nikodym derivative of ρ.Iic_snd
with respect to ρ.fst
at each
r : ℚ
. This function ℚ → α → ℝ≥0∞
is such that for almost all a : α
, the function ℚ → ℝ≥0∞
satisfies the properties of a cdf (monotone with limit 0 at -∞ and 1 at +∞, right-continuous).
We define this function on ℚ
and not ℝ
because ℚ
is countable, which allows us to prove
properties of the form ∀ᵐ a ∂ρ.fst, ∀ q, P (pre_cdf q a)
, instead of the weaker
∀ q, ∀ᵐ a ∂ρ.fst, P (pre_cdf q a)
.
- mono : monotone (λ (r : ℚ), probability_theory.pre_cdf ρ r a)
- le_one : ∀ (r : ℚ), probability_theory.pre_cdf ρ r a ≤ 1
- tendsto_at_top_one : filter.tendsto (λ (r : ℚ), probability_theory.pre_cdf ρ r a) filter.at_top (nhds 1)
- tendsto_at_bot_zero : filter.tendsto (λ (r : ℚ), probability_theory.pre_cdf ρ r a) filter.at_bot (nhds 0)
- infi_rat_gt_eq : ∀ (t : ℚ), (⨅ (r : ↥(set.Ioi t)), probability_theory.pre_cdf ρ ↑r a) = probability_theory.pre_cdf ρ t a
A product measure on α × ℝ
is said to have a conditional cdf at a : α
if pre_cdf
is
monotone with limit 0 at -∞ and 1 at +∞, and is right continuous.
This property holds almost everywhere (see has_cond_cdf_ae
).
A measurable set of elements of α
such that ρ
has a conditional cdf at all
a ∈ cond_cdf_set
.
Equations
- probability_theory.cond_cdf_set ρ = (measure_theory.to_measurable ρ.fst {b : α | ¬probability_theory.has_cond_cdf ρ b})ᶜ
Conditional cdf of the measure given the value on α
, restricted to the rationals.
It is defined to be pre_cdf
if a ∈ cond_cdf_set
, and a default cdf-like function
otherwise. This is an auxiliary definition used to define cond_cdf
.
Equations
- probability_theory.cond_cdf_rat ρ = λ (a : α), ite (a ∈ probability_theory.cond_cdf_set ρ) (λ (r : ℚ), (probability_theory.pre_cdf ρ r a).to_real) (λ (r : ℚ), ite (r < 0) 0 1)
Conditional cdf of the measure given the value on α
, as a plain function. This is an auxiliary
definition used to define cond_cdf
.
Equations
- probability_theory.cond_cdf' ρ = λ (a : α) (t : ℝ), ⨅ (r : {r' // t < ↑r'}), probability_theory.cond_cdf_rat ρ a ↑r
Conditional cdf #
Conditional cdf of the measure given the value on α
, as a Stieltjes function.
Equations
- probability_theory.cond_cdf ρ a = {to_fun := probability_theory.cond_cdf' ρ a, mono' := _, right_continuous' := _}
The conditional cdf is non-negative for all a : α
.
The conditional cdf is lower or equal to 1 for all a : α
.
The conditional cdf tends to 0 at -∞ for all a : α
.
The conditional cdf tends to 1 at +∞ for all a : α
.
The conditional cdf is a measurable function of a : α
for all x : ℝ
.
Auxiliary lemma for set_lintegral_cond_cdf
.
The conditional cdf is a strongly measurable function of a : α
for all x : ℝ
.
The function a ↦ (cond_cdf ρ a).measure
is measurable.