Filtration and stopping time #
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 is the first step in formalizing stochastic processes.
Main definitions #
measure_theory.filtration
: a filtration on a measurable spacemeasure_theory.adapted
: a sequence of functionsu
is said to be adapted to a filtrationf
if at each point in timei
,u i
isf i
-measurablemeasure_theory.filtration.natural
: the natural filtration with respect to a sequence of measurable functions is the smallest filtration to which it is adapted tomeasure_theory.is_stopping_time
: a stopping time with respect to some filtrationf
is a functionτ
such that for alli
, the preimage of{j | j ≤ i}
alongτ
isf i
-measurablemeasure_theory.is_stopping_time.measurable_space
: the σ-algebra associated with a stopping time
Tags #
filtration, stopping time, stochastic process
- seq : ι → measurable_space α
- mono : monotone self.seq
- le : ∀ (i : ι), self.seq i ≤ m
A filtration
on measurable space α
with σ-algebra m
is a monotone
sequence of of sub-σ-algebras of m
.
Equations
- measure_theory.filtration.has_coe_to_fun = {coe := λ (f : measure_theory.filtration ι m), f.seq}
The constant filtration which is equal to m
for all i : ι
.
Equations
- sigma_finite : ∀ (i : ι), measure_theory.sigma_finite (μ.trim _)
A measure is σ-finite with respect to filtration if it is σ-finite with respect to all the sub-σ-algebra of the filtration.
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 : ι), measurable (u i)
Given a sequence of functions, the natural filtration is the smallest sequence of σ-algebras such that that sequence of functions is measurable with respect to the filtration.
Equations
- measure_theory.filtration.natural u hum = {seq := λ (i : ι), ⨆ (j : ι) (H : j ≤ i), measurable_space.comap (u j) infer_instance, mono := _, le := _}
A stopping time with respect to some filtration f
is a function
τ
such that for all i
, the preimage of {j | j ≤ i}
along τ
is measurable
with respect to f i
.
Intuitively, the stopping time τ
describes some stopping rule such that at time
i
, we may determine it with the information we have at time i
.
Equations
- measure_theory.is_stopping_time f τ = ∀ (i : ι), measurable_set {x : α | τ x ≤ i}
The associated σ-algebra with a stopping time.
Equations
- hτ.measurable_space = {measurable_set' := λ (s : set α), ∀ (i : ι), measurable_set (s ∩ {x : α | τ x ≤ i}), measurable_set_empty := _, measurable_set_compl := _, measurable_set_Union := _}
Given a map u : ι → α → E
, its stopped value with respect to the stopping
time τ
is the map x ↦ u (τ x) x
.
Equations
- measure_theory.stopped_value u τ = λ (x : α), u (τ x) x
Given a map u : ι → α → E
, the stopped process with respect to τ
is u i x
if
i ≤ τ x
, and u (τ x) x
otherwise.
Intuitively, the stopped process stops evolving once the stopping time has occured.
Equations
- measure_theory.stopped_process u τ = λ (i : ι) (x : α), u (min i (τ x)) x