Integration in Probability Theory #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Integration results for independent random variables. Specifically, for two
independent random variables X and Y over the extended non-negative
reals, E[X * Y] = E[X] * E[Y]
, and similar results.
Implementation notes #
Many lemmas in this file take two arguments of the same typeclass. It is worth remembering that lean
will always pick the later typeclass in this situation, and does not care whether the arguments are
[]
, {}
, or ()
. All of these use the measurable_space
M2
to define μ
:
example {M1 : measurable_space Ω} [M2 : measurable_space Ω] {μ : measure Ω} : sorry := sorry
example [M1 : measurable_space Ω] {M2 : measurable_space Ω} {μ : measure Ω} : sorry := sorry
If a random variable f
in ℝ≥0∞
is independent of an event T
, then if you restrict the
random variable to T
, then E[f * indicator T c 0]=E[f] * E[indicator T c 0]
. It is useful for
lintegral_mul_eq_lintegral_mul_lintegral_of_independent_measurable_space
.
If f
and g
are independent random variables with values in ℝ≥0∞
,
then E[f * g] = E[f] * E[g]
. However, instead of directly using the independence
of the random variables, it uses the independence of measurable spaces for the
domains of f
and g
. This is similar to the sigma-algebra approach to
independence. See lintegral_mul_eq_lintegral_mul_lintegral_of_independent_fn
for
a more common variant of the product of independent variables.
If f
and g
are independent random variables with values in ℝ≥0∞
,
then E[f * g] = E[f] * E[g]
.
If f
and g
with values in ℝ≥0∞
are independent and almost everywhere measurable,
then E[f * g] = E[f] * E[g]
(slightly generalizing
lintegral_mul_eq_lintegral_mul_lintegral_of_indep_fun
).
The product of two independent, integrable, real_valued random variables is integrable.
If the product of two independent real_valued random variables is integrable and the second one is not almost everywhere zero, then the first one is integrable.
If the product of two independent real_valued random variables is integrable and the first one is not almost everywhere zero, then the second one is integrable.
The (Bochner) integral of the product of two independent, nonnegative random
variables is the product of their integrals. The proof is just plumbing around
lintegral_mul_eq_lintegral_mul_lintegral_of_indep_fun'
.
The (Bochner) integral of the product of two independent, integrable random
variables is the product of their integrals. The proof is pedestrian decomposition
into their positive and negative parts in order to apply indep_fun.integral_mul_of_nonneg
four times.
The (Bochner) integral of the product of two independent random variables is the product of their integrals.
Independence of functions f
and g
into arbitrary types is characterized by the relation
E[(φ ∘ f) * (ψ ∘ g)] = E[φ ∘ f] * E[ψ ∘ g]
for all measurable φ
and ψ
with values in ℝ
satisfying appropriate integrability conditions.