mathlib3 documentation

probability.process.filtration

Filtrations #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines filtrations of a measurable space and σ-finite filtrations.

Main definitions #

Main results #

Tags #

filtration, stochastic process

structure measure_theory.filtration {Ω : Type u_1} (ι : Type u_2) [preorder ι] (m : measurable_space Ω) :
Type (max u_1 u_2)

A filtration on a measurable space Ω with σ-algebra m is a monotone sequence of sub-σ-algebras of m.

Instances for measure_theory.filtration
@[protected]
theorem measure_theory.filtration.mono {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {i j : ι} (f : measure_theory.filtration ι m) (hij : i j) :
f i f j
@[protected]
theorem measure_theory.filtration.le {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] (f : measure_theory.filtration ι m) (i : ι) :
f i m
@[protected, ext]
theorem measure_theory.filtration.ext {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {f g : measure_theory.filtration ι m} (h : f = g) :
f = g
def measure_theory.filtration.const {Ω : Type u_1} (ι : Type u_3) {m : measurable_space Ω} [preorder ι] (m' : measurable_space Ω) (hm' : m' m) :

The constant filtration which is equal to m for all i : ι.

Equations
@[simp]
theorem measure_theory.filtration.const_apply {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {m' : measurable_space Ω} {hm' : m' m} (i : ι) :
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[norm_cast]
theorem measure_theory.filtration.coe_fn_sup {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {f g : measure_theory.filtration ι m} :
(f g) = f g
@[protected, instance]
Equations
@[norm_cast]
theorem measure_theory.filtration.coe_fn_inf {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {f g : measure_theory.filtration ι m} :
(f g) = f g
@[protected, instance]
Equations
theorem measure_theory.filtration.Sup_def {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] (s : set (measure_theory.filtration ι m)) (i : ι) :
@[protected, instance]
noncomputable def measure_theory.filtration.has_Inf {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] :
Equations
theorem measure_theory.filtration.Inf_def {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] (s : set (measure_theory.filtration ι m)) (i : ι) :
theorem measure_theory.measurable_set_of_filtration {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {f : measure_theory.filtration ι m} {s : set Ω} {i : ι} (hs : measurable_set s) :
@[class]
structure measure_theory.sigma_finite_filtration {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] (μ : measure_theory.measure Ω) (f : measure_theory.filtration ι m) :
Prop

A measure is σ-finite with respect to filtration if it is σ-finite with respect to all the sub-σ-algebra of the filtration.

Instances of this typeclass

Given a integrable function g, the conditional expectations of g with respect to a filtration is uniformly integrable.

def measure_theory.filtration_of_set {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {s : ι set Ω} (hsm : (i : ι), measurable_set (s i)) :

Given a sequence of measurable sets (sₙ), filtration_of_set is the smallest filtration such that sₙ is measurable with respect to the n-the sub-σ-algebra in filtration_of_set.

Equations
theorem measure_theory.measurable_set_filtration_of_set {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {s : ι set Ω} (hsm : (i : ι), measurable_set (s i)) (i : ι) {j : ι} (hj : j i) :
theorem measure_theory.measurable_set_filtration_of_set' {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {s : ι set Ω} (hsm : (n : ι), measurable_set (s n)) (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
noncomputable def measure_theory.filtration.limit_process {Ω : Type u_1} {ι : Type u_3} {m : measurable_space Ω} [preorder ι] {E : Type u_4} [has_zero E] [topological_space E] (f : ι Ω E) (ℱ : measure_theory.filtration ι m) (μ : measure_theory.measure Ω . "volume_tac") :
Ω E

Given a process f and a filtration , if f converges to some g almost everywhere and g is ⨆ n, ℱ n-measurable, then limit_process f ℱ μ chooses said g, else it returns 0.

This definition is used to phrase the a.e. martingale convergence theorem submartingale.ae_tendsto_limit_process where an L¹-bounded submartingale f adapted to converges to limit_process f ℱ μ μ-almost everywhere.

Equations