Centering lemma for stochastic processes #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Any ℕ
-indexed stochastic process which is adapted and integrable can be written as the sum of a
martingale and a predictable process. This result is also known as Doob's decomposition theorem.
From a process f
, a filtration ℱ
and a measure μ
, we define two processes
martingale_part f ℱ μ
and predictable_part f ℱ μ
.
Main definitions #
measure_theory.predictable_part f ℱ μ
: a predictable process such thatf = predictable_part f ℱ μ + martingale_part f ℱ μ
measure_theory.martingale_part f ℱ μ
: a martingale such thatf = predictable_part f ℱ μ + martingale_part f ℱ μ
Main statements #
measure_theory.adapted_predictable_part
:(λ n, predictable_part f ℱ μ (n+1))
is adapted. That is,predictable_part
is predictable.measure_theory.martingale_martingale_part
:martingale_part f ℱ μ
is a martingale.
Any ℕ
-indexed stochastic process can be written as the sum of a martingale and a predictable
process. This is the predictable process. See martingale_part
for the martingale.
Equations
- measure_theory.predictable_part f ℱ μ = λ (n : ℕ), (finset.range n).sum (λ (i : ℕ), measure_theory.condexp (⇑ℱ i) μ (f (i + 1) - f i))
Any ℕ
-indexed stochastic process can be written as the sum of a martingale and a predictable
process. This is the martingale. See predictable_part
for the predictable process.
Equations
- measure_theory.martingale_part f ℱ μ = λ (n : ℕ), f n - measure_theory.predictable_part f ℱ μ n