File tree Expand file tree Collapse file tree 2 files changed +6
-7
lines changed Expand file tree Collapse file tree 2 files changed +6
-7
lines changed Original file line number Diff line number Diff line change @@ -87,13 +87,6 @@ theorem atTop_le_nhds_top {α : Type*} [TopologicalSpace α] [LinearOrder α] [O
8787 @atBot_le_nhds_bot αᵒᵈ _ _ _ _
8888#align at_top_le_nhds_top atTop_le_nhds_top
8989
90- -- todo: move to topology/algebra/order/monotone_convergence
91- theorem tendsto_of_antitone {ι α : Type *} [Preorder ι] [TopologicalSpace α]
92- [ConditionallyCompleteLinearOrder α] [OrderTopology α] {f : ι → α} (h_mono : Antitone f) :
93- Tendsto f atTop atBot ∨ ∃ l, Tendsto f atTop (𝓝 l) :=
94- @tendsto_of_monotone ι αᵒᵈ _ _ _ _ _ h_mono
95- #align tendsto_of_antitone tendsto_of_antitone
96-
9790-- todo: move to measure_theory/measurable_space
9891/-- Monotone convergence for an infimum over a directed family and indexed by a countable type -/
9992theorem lintegral_iInf_directed_of_measurable {mα : MeasurableSpace α} [Countable β]
Original file line number Diff line number Diff line change @@ -227,6 +227,12 @@ theorem tendsto_of_monotone {ι α : Type*} [Preorder ι] [TopologicalSpace α]
227227 else Or.inl <| tendsto_atTop_atTop_of_monotone' h_mono H
228228#align tendsto_of_monotone tendsto_of_monotone
229229
230+ theorem tendsto_of_antitone {ι α : Type *} [Preorder ι] [TopologicalSpace α]
231+ [ConditionallyCompleteLinearOrder α] [OrderTopology α] {f : ι → α} (h_mono : Antitone f) :
232+ Tendsto f atTop atBot ∨ ∃ l, Tendsto f atTop (𝓝 l) :=
233+ @tendsto_of_monotone ι αᵒᵈ _ _ _ _ _ h_mono
234+ #align tendsto_of_antitone tendsto_of_antitone
235+
230236theorem tendsto_iff_tendsto_subseq_of_monotone {ι₁ ι₂ α : Type *} [SemilatticeSup ι₁] [Preorder ι₂]
231237 [Nonempty ι₁] [TopologicalSpace α] [ConditionallyCompleteLinearOrder α] [OrderTopology α]
232238 [NoMaxOrder α] {f : ι₂ → α} {φ : ι₁ → ι₂} {l : α} (hf : Monotone f)
You can’t perform that action at this time.
0 commit comments