Stopping times, stopped processes and stopped values #
Definition and properties of stopping times.
Main definitions #
MeasureTheory.IsStoppingTime
: a stopping time with respect to some filtrationf
is a functionτ
such that for alli
, the preimage of{j | j ≤ i}
alongτ
isf i
-measurableMeasureTheory.IsStoppingTime.measurableSpace
: the σ-algebra associated with a stopping time
Main results #
ProgMeasurable.stoppedProcess
: the stopped process of a progressively measurable process is progressively measurable.memℒp_stoppedProcess
: 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
- MeasureTheory.IsStoppingTime f τ = ∀ (i : ι), MeasurableSet {ω : Ω | τ ω ≤ i}
Instances For
Auxiliary lemma for MeasureTheory.IsStoppingTime.measurableSet_lt
.
The associated σ-algebra with a stopping time.
Equations
- hτ.measurableSpace = { MeasurableSet' := fun (s : Set Ω) => ∀ (i : ι), MeasurableSet (s ∩ {ω : Ω | τ ω ≤ i}), measurableSet_empty := ⋯, measurableSet_compl := ⋯, measurableSet_iUnion := ⋯ }
Instances For
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Stopped value and stopped process #
Given a map u : ι → Ω → E
, its stopped value with respect to the stopping
time τ
is the map x ↦ u (τ ω) ω
.
Equations
- MeasureTheory.stoppedValue u τ ω = u (τ ω) ω
Instances For
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 occurred.
Equations
- MeasureTheory.stoppedProcess u τ i ω = u (i ⊓ τ ω) ω
Instances For
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.