Stopping times, stopped processes and stopped values #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Definition and properties of stopping times.
Main definitions #
measure_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
Main results #
prog_measurable.stopped_process
: the stopped process of a progressively measurable process is progressively measurable.mem_ℒp_stopped_process
: if a process belongs toℒp
at every time inℕ
, then its stopped process belongs toℒp
as well.
Tags #
stopping time, stochastic process
Stopping times #
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 {ω : Ω | τ ω ≤ i}
Auxiliary lemma for is_stopping_time.measurable_set_lt
.
The associated σ-algebra with a stopping time.
Equations
- hτ.measurable_space = {measurable_set' := λ (s : set Ω), ∀ (i : ι), measurable_set (s ∩ {ω : Ω | τ ω ≤ i}), measurable_set_empty := _, measurable_set_compl := _, measurable_set_Union := _}
Stopped value and stopped process #
Given a map u : ι → Ω → E
, the stopped process with respect to τ
is u i ω
if
i ≤ τ ω
, and u (τ ω) ω
otherwise.
Intuitively, the stopped process stops evolving once the stopping time has occured.
Equations
- measure_theory.stopped_process u τ = λ (i : ι) (ω : Ω), u (linear_order.min i (τ ω)) ω
The stopped process of an adapted process with continuous paths is adapted.
If the indexing order has the discrete topology, then the stopped process of an adapted process is adapted.
Filtrations indexed by ℕ
#
Given stopping times τ
and η
which are bounded below, set.piecewise s τ η
is also
a stopping time with respect to the same filtration.