Documentation

Mathlib.Probability.Process.PartitionFiltration

Filtration built from the finite partitions of a countably generated measurable space #

In a countably generated measurable space α, we can build a sequence of finer and finer finite measurable partitions of the space such that the measurable space is generated by the union of all partitions. This sequence of partitions is defined in MeasureTheory.MeasurableSpace.CountablyGenerated.

Here, we build the filtration of the measurable spaces generated by countablePartition α n for all n : ℕ, which we call countableFiltration α. Since each measurable space in the filtration is finite, we can easily build measurable functions on those spaces. A potential application of countableFiltration α is to build a martingale with respect to that filtration and use the martingale convergence theorems to define a measurable function on α.

Main definitions #

Main statements #

def ProbabilityTheory.partitionFiltration {α : Type u_1} [m : MeasurableSpace α] {t : Set α} (ht : ∀ (n : ), MeasurableSet (t n)) :

A filtration built from the measurable spaces generated by the partitions memPartition t n for all n : ℕ.

Equations
Instances For
    theorem ProbabilityTheory.measurableSet_partitionFiltration_of_mem {α : Type u_1} [m : MeasurableSpace α] {t : Set α} (ht : ∀ (n : ), MeasurableSet (t n)) (n : ) {s : Set α} (hs : s memPartition t n) :
    theorem ProbabilityTheory.measurableSet_partitionFiltration_memPartitionSet {α : Type u_1} [m : MeasurableSpace α] {t : Set α} (ht : ∀ (n : ), MeasurableSet (t n)) (n : ) (a : α) :
    theorem ProbabilityTheory.measurable_memPartitionSet_subtype {α : Type u_1} [m : MeasurableSpace α] {t : Set α} (ht : ∀ (n : ), MeasurableSet (t n)) (n : ) (m : MeasurableSpace (memPartition t n)) :
    Measurable fun (a : α) => memPartitionSet t n a,
    theorem ProbabilityTheory.measurable_memPartitionSet {α : Type u_1} [m : MeasurableSpace α] {t : Set α} (ht : ∀ (n : ), MeasurableSet (t n)) (n : ) :
    theorem ProbabilityTheory.iSup_partitionFiltration {α : Type u_1} [m : MeasurableSpace α] {t : Set α} (ht : ∀ (n : ), MeasurableSet (t n)) (ht_range : MeasurableSpace.generateFrom (Set.range t) = m) :

    A filtration built from the measurable spaces generated by countablePartition α n for all n : ℕ.

    Equations
    Instances For