Documentation

Mathlib.MeasureTheory.Constructions.BorelSpace.WithTop

Borel measurable space on WithTop #

For ι a linear order with the order topology, we define the Borel measurable space on WithTop ι. We then prove that the natural inclusion ι → WithTop ι is measurable, and that the function WithTop.untopA : WithTop ι → ι (which sends to an arbitrary element of ι) is measurable.

Main statements #

Measurable equivalence between the non-top elements of WithTop ι and ι.

Equations
Instances For
    theorem WithTop.measurable_of_measurable_comp_coe {ι : Type u_1} [LinearOrder ι] [TopologicalSpace ι] [OrderTopology ι] [MeasurableSpace ι] [BorelSpace ι] {α : Type u_2} { : MeasurableSpace α} {f : WithTop ια} (h : Measurable fun (p : ι) => f p) :
    theorem WithTop.measurable_coe {ι : Type u_1} [LinearOrder ι] [TopologicalSpace ι] [OrderTopology ι] [MeasurableSpace ι] [BorelSpace ι] :
    Measurable fun (x : ι) => x
    theorem Measurable.withTop_coe {ι : Type u_1} [LinearOrder ι] [TopologicalSpace ι] [OrderTopology ι] [MeasurableSpace ι] [BorelSpace ι] {α : Type u_2} { : MeasurableSpace α} {f : αι} (hf : Measurable f) :
    Measurable fun (x : α) => (f x)
    theorem Measurable.untopD {ι : Type u_1} [LinearOrder ι] [TopologicalSpace ι] [OrderTopology ι] [MeasurableSpace ι] [BorelSpace ι] {α : Type u_2} { : MeasurableSpace α} (d : ι) {f : αWithTop ι} (hf : Measurable f) :
    Measurable fun (x : α) => WithTop.untopD d (f x)
    theorem Measurable.untopA {ι : Type u_1} [LinearOrder ι] [TopologicalSpace ι] [OrderTopology ι] [MeasurableSpace ι] [BorelSpace ι] {α : Type u_2} { : MeasurableSpace α} [Nonempty ι] {f : αWithTop ι} (hf : Measurable f) :
    Measurable fun (x : α) => (f x).untopA

    Measurable equivalence between WithTop ι and ι ⊕ Unit.

    Equations
    Instances For