Documentation

Mathlib.Probability.Process.Predictable

Predictable σ-algebra #

This file defines the predictable σ-algebra associated to a filtration, as well as the notion of predictable processes. We prove that predictable processes are progressively measurable and adapted. We also give an equivalent characterization of predictability for discrete processes.

Main definitions #

Main results #

Tags #

predictable, previsible

def MeasureTheory.Filtration.predictable {Ω : Type u_1} {ι : Type u_2} {m : MeasurableSpace Ω} [Preorder ι] [OrderBot ι] (𝓕 : Filtration ι m) :

Given a filtration 𝓕, the predictable σ-algebra is the σ-algebra on ι × Ω generated by sets of the form (t, ∞) × A for t ∈ ι and A ∈ 𝓕 t and {⊥} × A for A ∈ 𝓕 ⊥.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def MeasureTheory.IsPredictable {Ω : Type u_1} {ι : Type u_2} {m : MeasurableSpace Ω} {E : Type u_3} [TopologicalSpace E] [Preorder ι] [OrderBot ι] (𝓕 : Filtration ι m) (u : ιΩE) :

    A process is said to be predictable if it is measurable with respect to the predictable σ-algebra.

    Equations
    Instances For
      theorem MeasureTheory.measurableSet_predictable_Ioi_prod {Ω : Type u_1} {ι : Type u_2} {m : MeasurableSpace Ω} [LinearOrder ι] [OrderBot ι] {𝓕 : Filtration ι m} {i : ι} {s : Set Ω} (hs : MeasurableSet s) :
      theorem MeasureTheory.measurableSet_predictable_Ioc_prod {Ω : Type u_1} {ι : Type u_2} {m : MeasurableSpace Ω} [LinearOrder ι] [OrderBot ι] {𝓕 : Filtration ι m} (i j : ι) {s : Set Ω} (hs : MeasurableSet s) :

      Sets of the form (i, j] × A for any A ∈ 𝓕 i are measurable with respect to the predictable σ-algebra.

      theorem MeasureTheory.measurableSpace_le_predictable_of_measurableSet {Ω : Type u_1} {ι : Type u_2} {m : MeasurableSpace Ω} [Preorder ι] [OrderBot ι] {𝓕 : Filtration ι m} {m' : MeasurableSpace (ι × Ω)} (hm'bot : ∀ (A : Set Ω), MeasurableSet AMeasurableSet ({} ×ˢ A)) (hm' : ∀ (i : ι) (A : Set Ω), MeasurableSet AMeasurableSet (Set.Ioi i ×ˢ A)) :

      A predictable process is progressively measurable.

      A predictable process is adapted.

      theorem MeasureTheory.IsPredictable.measurable_add_one {Ω : Type u_1} {m : MeasurableSpace Ω} {E : Type u_3} [TopologicalSpace E] [TopologicalSpace.MetrizableSpace E] [MeasurableSpace E] [BorelSpace E] {𝓕 : Filtration m} {u : ΩE} (h𝓕 : IsPredictable 𝓕 u) (n : ) :
      Measurable (u (n + 1))

      If u is a discrete predictable process, then u (n + 1) is 𝓕 n-measurable.

      theorem MeasureTheory.isPredictable_of_measurable_add_one {Ω : Type u_1} {m : MeasurableSpace Ω} {E : Type u_3} [TopologicalSpace E] [TopologicalSpace.MetrizableSpace E] [MeasurableSpace E] [BorelSpace E] [SecondCountableTopology E] {𝓕 : Filtration m} {u : ΩE} (h₀ : Measurable (u 0)) (h : ∀ (n : ), Measurable (u (n + 1))) :

      A discrete process u is predictable iff u (n + 1) is 𝓕 n-measurable for all n and u 0 is 𝓕 0-measurable.