Adapted and progressively measurable processes #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines some standard definition from the theory of stochastic processes including filtrations and stopping times. These definitions are used to model the amount of information at a specific time and are the first step in formalizing stochastic processes.
Main definitions #
measure_theory.adapted
: a sequence of functionsu
is said to be adapted to a filtrationf
if at each point in timei
,u i
isf i
-strongly measurablemeasure_theory.prog_measurable
: a sequence of functionsu
is said to be progressively measurable with respect to a filtrationf
if at each point in timei
,u
restricted toset.Iic i × Ω
is strongly measurable with respect to the productmeasurable_space
structure where the σ-algebra used forΩ
isf i
.
Main results #
adapted.prog_measurable_of_continuous
: a continuous adapted process is progressively measurable.
Tags #
adapted, progressively measurable
A sequence of functions u
is adapted to a filtration f
if for all i
,
u i
is f i
-measurable.
Equations
- measure_theory.adapted f u = ∀ (i : ι), measure_theory.strongly_measurable (u i)
Progressively measurable process. A sequence of functions u
is said to be progressively
measurable with respect to a filtration f
if at each point in time i
, u
restricted to
set.Iic i × Ω
is measurable with respect to the product measurable_space
structure where the
σ-algebra used for Ω
is f i
.
The usual definition uses the interval [0,i]
, which we replace by set.Iic i
. We recover the
usual definition for index types ℝ≥0
or ℕ
.
Equations
- measure_theory.prog_measurable f u = ∀ (i : ι), measure_theory.strongly_measurable (λ (p : ↥(set.Iic i) × Ω), u ↑(p.fst) p.snd)
A continuous and adapted process is progressively measurable.
For filtrations indexed by a discrete order, adapted
and prog_measurable
are equivalent.
This lemma provides adapted f u → prog_measurable f u
.
See prog_measurable.adapted
for the reverse direction, which is true more generally.