Documentation

Mathlib.Topology.Order.LowerUpperTopology

Lower and Upper topology #

This file introduces the lower topology on a preorder as the topology generated by the complements of the left-closed right-infinite intervals.

For completeness we also introduce the dual upper topology, generated by the complements of the right-closed left-infinite intervals.

Main statements #

Implementation notes #

A type synonym WithLower is introduced and for a preorder α, WithLower α is made an instance of TopologicalSpace by the topology generated by the complements of the closed intervals to infinity.

We define a mixin class IsLower for the class of types which are both a preorder and a topology and where the topology is generated by the complements of the closed intervals to infinity. It is shown that WithLower α is an instance of IsLower.

Similarly for the upper topology.

Motivation #

The lower topology is used with the Scott topology to define the Lawson topology. The restriction of the lower topology to the spectrum of a complete lattice coincides with the hull-kernel topology.

References #

Tags #

lower topology, upper topology, preorder

The lower topology is the topology generated by the complements of the left-closed right-infinite intervals.

Equations
Instances For

    The upper topology is the topology generated by the complements of the right-closed left-infinite intervals.

    Equations
    Instances For
      def Topology.WithLower (α : Type u_1) :
      Type u_1

      Type synonym for a preorder equipped with the lower set topology.

      Equations
      Instances For
        @[match_pattern]

        toLower is the identity function to the WithLower of a type.

        Equations
        Instances For
          @[match_pattern]

          ofLower is the identity function from the WithLower of a type.

          Equations
          Instances For
            @[deprecated Topology.WithLower.toLower_symm (since := "2024-12-16")]

            Alias of Topology.WithLower.toLower_symm.

            @[deprecated Topology.WithLower.ofLower_symm (since := "2024-12-16")]

            Alias of Topology.WithLower.ofLower_symm.

            @[simp]
            theorem Topology.WithLower.toLower_ofLower {α : Type u_1} (a : WithLower α) :
            toLower (ofLower a) = a
            @[simp]
            theorem Topology.WithLower.ofLower_toLower {α : Type u_1} (a : α) :
            ofLower (toLower a) = a
            theorem Topology.WithLower.toLower_inj {α : Type u_1} {a b : α} :
            toLower a = toLower b a = b
            theorem Topology.WithLower.ofLower_inj {α : Type u_1} {a b : WithLower α} :
            ofLower a = ofLower b a = b
            def Topology.WithLower.rec {α : Type u_1} {β : WithLower αSort u_3} (h : (a : α) → β (toLower a)) (a : WithLower α) :
            β a

            A recursor for WithLower. Use as induction x.

            Equations
            Instances For
              @[simp]
              theorem Topology.WithLower.toLower_le_toLower {α : Type u_1} [Preorder α] {x y : α} :
              toLower x toLower y x y
              @[simp]
              theorem Topology.WithLower.toLower_lt_toLower {α : Type u_1} [Preorder α] {x y : α} :
              toLower x < toLower y x < y
              @[simp]
              theorem Topology.WithLower.ofLower_le_ofLower {α : Type u_1} [Preorder α] {x y : WithLower α} :
              ofLower x ofLower y x y
              @[simp]
              theorem Topology.WithLower.ofLower_lt_ofLower {α : Type u_1} [Preorder α] {x y : WithLower α} :
              ofLower x < ofLower y x < y
              def Topology.WithUpper (α : Type u_3) :
              Type u_3

              Type synonym for a preorder equipped with the upper topology.

              Equations
              Instances For
                @[match_pattern]

                toUpper is the identity function to the WithUpper of a type.

                Equations
                Instances For
                  @[match_pattern]

                  ofUpper is the identity function from the WithUpper of a type.

                  Equations
                  Instances For
                    @[deprecated Topology.WithUpper.toUpper_symm (since := "2024-12-16")]

                    Alias of Topology.WithUpper.toUpper_symm.

                    @[deprecated Topology.WithUpper.ofUpper_symm (since := "2024-12-16")]

                    Alias of Topology.WithUpper.ofUpper_symm.

                    @[simp]
                    theorem Topology.WithUpper.toUpper_ofUpper {α : Type u_1} (a : WithUpper α) :
                    toUpper (ofUpper a) = a
                    @[simp]
                    theorem Topology.WithUpper.ofUpper_toUpper {α : Type u_1} (a : α) :
                    ofUpper (toUpper a) = a
                    theorem Topology.WithUpper.toUpper_inj {α : Type u_1} {a b : α} :
                    toUpper a = toUpper b a = b
                    theorem Topology.WithUpper.ofUpper_inj {α : Type u_1} {a b : WithUpper α} :
                    ofUpper a = ofUpper b a = b
                    def Topology.WithUpper.rec {α : Type u_1} {β : WithUpper αSort u_3} (h : (a : α) → β (toUpper a)) (a : WithUpper α) :
                    β a

                    A recursor for WithUpper. Use as induction x.

                    Equations
                    Instances For
                      @[simp]
                      theorem Topology.WithUpper.toUpper_le_toUpper {α : Type u_1} [Preorder α] {x y : α} :
                      toUpper x toUpper y x y
                      @[simp]
                      theorem Topology.WithUpper.toUpper_lt_toUpper {α : Type u_1} [Preorder α] {x y : α} :
                      toUpper x < toUpper y x < y
                      @[simp]
                      theorem Topology.WithUpper.ofUpper_le_ofUpper {α : Type u_1} [Preorder α] {x y : WithUpper α} :
                      ofUpper x ofUpper y x y
                      @[simp]
                      theorem Topology.WithUpper.ofUpper_lt_ofUpper {α : Type u_1} [Preorder α] {x y : WithUpper α} :
                      ofUpper x < ofUpper y x < y
                      class Topology.IsLower (α : Type u_3) [t : TopologicalSpace α] [Preorder α] :

                      The lower topology is the topology generated by the complements of the left-closed right-infinite intervals.

                      • topology_eq_lowerTopology : t = lower α
                      Instances
                        class Topology.IsUpper (α : Type u_3) [t : TopologicalSpace α] [Preorder α] :

                        The upper topology is the topology generated by the complements of the right-closed left-infinite intervals.

                        • topology_eq_upperTopology : t = upper α
                        Instances

                          The lower topology is homeomorphic to the upper topology on the dual order

                          Equations
                          Instances For
                            def Topology.IsLower.lowerBasis (α : Type u_3) [Preorder α] :
                            Set (Set α)

                            The complements of the upper closures of finite sets are a collection of lower sets which form a basis for the lower topology.

                            Equations
                            Instances For
                              theorem Topology.IsLower.topology_eq (α : Type u_1) [Preorder α] [TopologicalSpace α] [IsLower α] :
                              inst✝ = lower α

                              If α is equipped with the lower topology, then it is homeomorphic to WithLower α.

                              Equations
                              Instances For

                                Left-closed right-infinite intervals [a, ∞) are closed in the lower topology.

                                theorem Topology.IsLower.isClosed_upperClosure {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsLower α] {s : Set α} (h : s.Finite) :

                                The upper closure of a finite set is closed in the lower topology.

                                theorem Topology.IsLower.isLowerSet_of_isOpen {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsLower α] {s : Set α} (h : IsOpen s) :

                                Every set open in the lower topology is a lower set.

                                theorem Topology.IsLower.tendsto_nhds_iff_not_le {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsLower α] {β : Type u_3} {f : βα} {l : Filter β} {x : α} :
                                Filter.Tendsto f l (nhds x) ∀ (y : α), ¬y x∀ᶠ (z : β) in l, ¬y f z
                                @[simp]
                                theorem Topology.IsLower.closure_singleton {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsLower α] (a : α) :

                                The closure of a singleton {a} in the lower topology is the left-closed right-infinite interval [a, ∞).

                                theorem Topology.IsLower.continuous_iff_Ici {α : Type u_1} {β : Type u_2} [Preorder α] [TopologicalSpace α] [IsLower α] [TopologicalSpace β] {f : βα} :
                                Continuous f ∀ (a : α), IsClosed (f ⁻¹' Set.Ici a)

                                A function f : β → α with lower topology in the codomain is continuous if and only if the preimage of every interval Set.Ici a is a closed set.

                                @[instance 90]

                                The lower topology on a partial order is T₀.

                                theorem Topology.IsLower.tendsto_nhds_iff_lt {α : Type u_1} [LinearOrder α] [TopologicalSpace α] [IsLower α] {β : Type u_3} {f : βα} {l : Filter β} {x : α} :
                                Filter.Tendsto f l (nhds x) ∀ (y : α), x < y∀ᶠ (z : β) in l, f z < y
                                def Topology.IsUpper.upperBasis (α : Type u_3) [Preorder α] :
                                Set (Set α)

                                The complements of the lower closures of finite sets are a collection of upper sets which form a basis for the upper topology.

                                Equations
                                Instances For
                                  theorem Topology.IsUpper.topology_eq (α : Type u_1) [Preorder α] [TopologicalSpace α] [IsUpper α] :
                                  inst✝ = upper α

                                  If α is equipped with the upper topology, then it is homeomorphic to WithUpper α.

                                  Equations
                                  Instances For

                                    Left-infinite right-closed intervals (-∞,a] are closed in the upper topology.

                                    theorem Topology.IsUpper.isClosed_lowerClosure {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsUpper α] {s : Set α} (h : s.Finite) :

                                    The lower closure of a finite set is closed in the upper topology.

                                    theorem Topology.IsUpper.isUpperSet_of_isOpen {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsUpper α] {s : Set α} (h : IsOpen s) :

                                    Every set open in the upper topology is a upper set.

                                    theorem Topology.IsUpper.tendsto_nhds_iff_not_le {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsUpper α] {β : Type u_3} {f : βα} {l : Filter β} {x : α} :
                                    Filter.Tendsto f l (nhds x) ∀ (y : α), ¬x y∀ᶠ (z : β) in l, ¬f z y
                                    @[simp]
                                    theorem Topology.IsUpper.closure_singleton {α : Type u_1} [Preorder α] [TopologicalSpace α] [IsUpper α] (a : α) :

                                    The closure of a singleton {a} in the upper topology is the left-infinite right-closed interval (-∞,a].

                                    theorem Topology.IsUpper.continuous_iff_Iic {α : Type u_1} {β : Type u_2} [Preorder α] [TopologicalSpace α] [IsUpper α] [TopologicalSpace β] {f : βα} :
                                    Continuous f ∀ (a : α), IsClosed (f ⁻¹' Set.Iic a)

                                    A function f : β → α with upper topology in the codomain is continuous if and only if the preimage of every interval Set.Iic a is a closed set.

                                    @[instance 90]

                                    The upper topology on a partial order is T₀.

                                    theorem Topology.IsUpper.tendsto_nhds_iff_lt {α : Type u_1} [LinearOrder α] [TopologicalSpace α] [IsUpper α] {β : Type u_3} {f : βα} {l : Filter β} {x : α} :
                                    Filter.Tendsto f l (nhds x) y < x, ∀ᶠ (z : β) in l, y < f z
                                    instance Topology.instIsLowerProd {α : Type u_1} {β : Type u_2} [Preorder α] [TopologicalSpace α] [IsLower α] [OrderBot α] [Preorder β] [TopologicalSpace β] [IsLower β] [OrderBot β] :
                                    IsLower (α × β)
                                    instance Topology.instIsUpperProd {α : Type u_1} {β : Type u_2} [Preorder α] [TopologicalSpace α] [IsUpper α] [OrderTop α] [Preorder β] [TopologicalSpace β] [IsUpper β] [OrderTop β] :
                                    IsUpper (α × β)

                                    The Sierpiński topology on Prop is the upper topology