Skip to content

Commit

Permalink
feat(measure_theory/borel_space): a monotone function is measurable (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
ADedecker committed Jul 14, 2021
1 parent 8e5af43 commit 51cc43e
Showing 1 changed file with 16 additions and 1 deletion.
17 changes: 16 additions & 1 deletion src/measure_theory/borel_space.lean
Expand Up @@ -768,6 +768,21 @@ begin
exact ⟨hg.exists.some, hg.mono (λ y hy, is_glb.unique hy hg.exists.some_spec)⟩,
end

lemma measurable_of_monotone [linear_order β] [order_topology β] {f : β → α} (hf : monotone f) :
measurable f :=
suffices h : ∀ x, ord_connected (f ⁻¹' Ioi x),
from measurable_of_Ioi (λ x, (h x).measurable_set),
λ x, ord_connected_def.mpr (λ a ha b hb c hc, lt_of_lt_of_le ha (hf hc.1))

alias measurable_of_monotone ← monotone.measurable

lemma measurable_of_antimono [linear_order β] [order_topology β] {f : β → α}
(hf : ∀ ⦃x y : β⦄, x ≤ y → f y ≤ f x) :
measurable f :=
suffices h : ∀ x, ord_connected (f ⁻¹' Ioi x),
from measurable_of_Ioi (λ x, (h x).measurable_set),
λ x, ord_connected_def.mpr (λ a ha b hb c hc, lt_of_lt_of_le hb (hf hc.2))

end linear_order

@[measurability]
Expand Down Expand Up @@ -879,7 +894,7 @@ end complete_linear_order

section conditionally_complete_linear_order

variables [conditionally_complete_linear_order α] [second_countable_topology α] [order_topology α]
variables [conditionally_complete_linear_order α] [order_topology α] [second_countable_topology α]

lemma measurable_cSup {ι} {f : ι → δ → α} {s : set ι} (hs : s.countable)
(hf : ∀ i, measurable (f i)) (bdd : ∀ x, bdd_above ((λ i, f i x) '' s)) :
Expand Down

0 comments on commit 51cc43e

Please sign in to comment.