The strong law of large numbers #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We prove the strong law of large numbers, in probability_theory.strong_law_ae
:
If X n
is a sequence of independent identically distributed integrable real-valued random
variables, then ∑ i in range n, X i / n
converges almost surely to 𝔼[X 0]
.
We give here the strong version, due to Etemadi, that only requires pairwise independence.
This file also contains the Lᵖ version of the strong law of large numbers provided by
probability_theory.strong_law_Lp
which shows ∑ i in range n, X i / n
converges in Lᵖ to
𝔼[X 0]
provided X n
is independent identically distributed and is Lᵖ.
Implementation #
We follow the proof by Etemadi Etemadi, An elementary proof of the strong law of large numbers, which goes as follows.
It suffices to prove the result for nonnegative X
, as one can prove the general result by
splitting a general X
into its positive part and negative part.
Consider Xₙ
a sequence of nonnegative integrable identically distributed pairwise independent
random variables. Let Yₙ
be the truncation of Xₙ
up to n
. We claim that
- Almost surely,
Xₙ = Yₙ
for all but finitely many indices. Indeed,∑ ℙ (Xₙ ≠ Yₙ)
is bounded by1 + 𝔼[X]
(seesum_prob_mem_Ioc_le
andtsum_prob_mem_Ioi_lt_top
). - Let
c > 1
. Along the sequencen = c ^ k
, then(∑_{i=0}^{n-1} Yᵢ - 𝔼[Yᵢ])/n
converges almost surely to0
. This follows from a variance control, as
∑_k ℙ (|∑_{i=0}^{c^k - 1} Yᵢ - 𝔼[Yᵢ]| > c^k ε)
≤ ∑_k (c^k ε)^{-2} ∑_{i=0}^{c^k - 1} Var[Yᵢ] (by Markov inequality)
≤ ∑_i (C/i^2) Var[Yᵢ] (as ∑_{c^k > i} 1/(c^k)^2 ≤ C/i^2)
≤ ∑_i (C/i^2) 𝔼[Yᵢ^2]
≤ 2C 𝔼[X^2] (see `sum_variance_truncation_le`)
- As
𝔼[Yᵢ]
converges to𝔼[X]
, it follows from the two previous items and Cesaro that, along the sequencen = c^k
, one has(∑_{i=0}^{n-1} Xᵢ) / n → 𝔼[X]
almost surely. - To generalize it to all indices, we use the fact that
∑_{i=0}^{n-1} Xᵢ
is nondecreasing and that, ifc
is close enough to1
, the gap betweenc^k
andc^(k+1)
is small.
Prerequisites on truncations #
If a function is integrable, then the integral of its truncated versions converges to the integral of the whole function.
The expectation of the truncated version of Xᵢ
behaves asymptotically like the whole
expectation. This follows from convergence and Cesaro averaging.
The truncated and non-truncated versions of Xᵢ
have the same asymptotic behavior, as they
almost surely coincide at all but finitely many steps. This follows from a probability computation
and Borel-Cantelli.
Xᵢ
satisfies the strong law of large numbers along all integers. This follows from the
corresponding fact along the sequences c^n
, and the fact that any integer can be sandwiched
between c^n
and c^(n+1)
with comparably small error if c
is close enough to 1
(which is formalized in tendsto_div_of_monotone_of_tendsto_div_floor_pow
).
Strong law of large numbers, almost sure version: if X n
is a sequence of independent
identically distributed integrable real-valued random variables, then ∑ i in range n, X i / n
converges almost surely to 𝔼[X 0]
. We give here the strong version, due to Etemadi, that only
requires pairwise independence.
Strong law of large numbers, Lᵖ version: if X n
is a sequence of independent
identically distributed real-valued random variables in Lᵖ, then ∑ i in range n, X i / n
converges in Lᵖ to 𝔼[X 0]
.