Typeclasses for measurability of lattice operations #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define classes has_measurable_sup
and has_measurable_inf
and prove dot-style
lemmas (measurable.sup
, ae_measurable.sup
etc). For binary operations we define two typeclasses:
has_measurable_sup
says that both left and right sup are measurable;has_measurable_sup₂
says thatλ p : α × α, p.1 ⊔ p.2
is measurable,
and similarly for other binary operations. The reason for introducing these classes is that in case
of topological space α
equipped with the Borel σ
-algebra, instances for has_measurable_sup₂
etc require α
to have a second countable topology.
For instances relating, e.g., has_continuous_sup
to has_measurable_sup
see file
measure_theory.borel_space
.
Tags #
measurable function, lattice operation
- measurable_const_sup : ∀ (c : M), measurable (has_sup.sup c)
- measurable_sup_const : ∀ (c : M), measurable (λ (_x : M), _x ⊔ c)
We say that a type has_measurable_sup
if ((⊔) c)
and (⊔ c)
are measurable functions.
For a typeclass assuming measurability of uncurry (⊔)
see has_measurable_sup₂
.
Instances of this typeclass
- measurable_sup : measurable (λ (p : M × M), p.fst ⊔ p.snd)
We say that a type has_measurable_sup₂
if uncurry (⊔)
is a measurable functions.
For a typeclass assuming measurability of ((⊔) c)
and (⊔ c)
see has_measurable_sup
.
Instances of this typeclass
- measurable_const_inf : ∀ (c : M), measurable (has_inf.inf c)
- measurable_inf_const : ∀ (c : M), measurable (λ (_x : M), _x ⊓ c)
We say that a type has_measurable_inf
if ((⊓) c)
and (⊓ c)
are measurable functions.
For a typeclass assuming measurability of uncurry (⊓)
see has_measurable_inf₂
.
Instances of this typeclass
- measurable_inf : measurable (λ (p : M × M), p.fst ⊓ p.snd)
We say that a type has_measurable_inf₂
if uncurry (⊔)
is a measurable functions.
For a typeclass assuming measurability of ((⊔) c)
and (⊔ c)
see has_measurable_inf
.