Skip to content

Commit

Permalink
feat: port Topology.Algebra.Order.Filter (#2167)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Feb 10, 2023
1 parent ae5cd16 commit 0796b6a
Show file tree
Hide file tree
Showing 2 changed files with 47 additions and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -1012,6 +1012,7 @@ import Mathlib.Topology.Algebra.Order.Archimedean
import Mathlib.Topology.Algebra.Order.Compact
import Mathlib.Topology.Algebra.Order.ExtendFrom
import Mathlib.Topology.Algebra.Order.ExtrClosure
import Mathlib.Topology.Algebra.Order.Filter
import Mathlib.Topology.Algebra.Order.IntermediateValue
import Mathlib.Topology.Algebra.Order.LeftRight
import Mathlib.Topology.Algebra.Order.LiminfLimsup
Expand Down
46 changes: 46 additions & 0 deletions Mathlib/Topology/Algebra/Order/Filter.lean
@@ -0,0 +1,46 @@
/-
Copyright (c) 2022 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
! This file was ported from Lean 3 source module topology.algebra.order.filter
! leanprover-community/mathlib commit 98e83c3d541c77cdb7da20d79611a780ff8e7d90
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
import Mathlib.Topology.Order.Basic
import Mathlib.Topology.Filter

/-!
# Topology on filters of a space with order topology
In this file we prove that `𝓝 (f x)` tends to `𝓝 Filter.atTop` provided that `f` tends to
`Filter.atTop`, and similarly for `Filter.atBot`.
-/


open Topology

namespace Filter

variable {Ξ± X : Type _} [TopologicalSpace X] [PartialOrder X] [OrderTopology X]

protected theorem tendsto_nhds_atTop [NoMaxOrder X] : Tendsto 𝓝 (atTop : Filter X) (𝓝 atTop) :=
Filter.tendsto_nhds_atTop_iff.2 fun x => (eventually_gt_atTop x).mono fun _ => le_mem_nhds
#align filter.tendsto_nhds_at_top Filter.tendsto_nhds_atTop

protected theorem tendsto_nhds_atBot [NoMinOrder X] : Tendsto 𝓝 (atBot : Filter X) (𝓝 atBot) :=
@Filter.tendsto_nhds_atTop Xα΅’α΅ˆ _ _ _ _
#align filter.tendsto_nhds_at_bot Filter.tendsto_nhds_atBot

theorem Tendsto.nhds_atTop [NoMaxOrder X] {f : Ξ± β†’ X} {l : Filter Ξ±} (h : Tendsto f l atTop) :
Tendsto (𝓝 ∘ f) l (𝓝 atTop) :=
Filter.tendsto_nhds_atTop.comp h
#align filter.tendsto.nhds_at_top Filter.Tendsto.nhds_atTop

theorem Tendsto.nhds_atBot [NoMinOrder X] {f : Ξ± β†’ X} {l : Filter Ξ±} (h : Tendsto f l atBot) :
Tendsto (𝓝 ∘ f) l (𝓝 atBot) :=
@Tendsto.nhds_atTop Ξ± Xα΅’α΅ˆ _ _ _ _ _ _ h
#align filter.tendsto.nhds_at_bot Filter.Tendsto.nhds_atBot

end Filter

0 comments on commit 0796b6a

Please sign in to comment.