Documentation

Mathlib.Topology.Order.UpperLowerSetTopology

Upper and lower sets topologies #

This file introduces the upper set topology on a preorder as the topology where the open sets are the upper sets and the lower set topology on a preorder as the topology where the open sets are the lower sets.

In general the upper set topology does not coincide with the upper topology and the lower set topology does not coincide with the lower topology.

Main statements #

We provide the upper set topology in three ways (and similarly for the lower set topology):

Motivation #

An Alexandrov topology is a topology where the intersection of any collection of open sets is open. The upper set topology is an Alexandrov topology and, given any Alexandrov topological space, we can equip it with a preorder (namely the specialization preorder) whose upper set topology coincides with the original topology. See Topology.Specialization.

Tags #

upper set topology, lower set topology, preorder, Alexandrov

Topology whose open sets are upper sets.

Note: In general the upper set topology does not coincide with the upper topology.

Equations
Instances For

    Topology whose open sets are lower sets.

    Note: In general the lower set topology does not coincide with the lower topology.

    Equations
    Instances For
      def Topology.WithUpperSet (α : Type u_4) :
      Type u_4

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

      Equations
      Instances For
        @[match_pattern]

        toUpperSet is the identity function to the WithUpperSet of a type.

        Equations
        Instances For
          @[match_pattern]

          ofUpperSet is the identity function from the WithUpperSet of a type.

          Equations
          Instances For
            @[deprecated Topology.WithUpperSet.toUpperSet_symm (since := "2024-10-10")]

            Alias of Topology.WithUpperSet.toUpperSet_symm.

            @[deprecated Topology.WithUpperSet.ofUpperSet_symm (since := "2024-10-10")]

            Alias of Topology.WithUpperSet.ofUpperSet_symm.

            @[simp]
            theorem Topology.WithUpperSet.toUpperSet_ofUpperSet {α : Type u_1} (a : WithUpperSet α) :
            toUpperSet (ofUpperSet a) = a
            @[simp]
            theorem Topology.WithUpperSet.ofUpperSet_toUpperSet {α : Type u_1} (a : α) :
            ofUpperSet (toUpperSet a) = a
            theorem Topology.WithUpperSet.toUpperSet_inj {α : Type u_1} {a b : α} :
            toUpperSet a = toUpperSet b a = b
            theorem Topology.WithUpperSet.ofUpperSet_inj {α : Type u_1} {a b : WithUpperSet α} :
            ofUpperSet a = ofUpperSet b a = b
            def Topology.WithUpperSet.rec {α : Type u_1} {β : WithUpperSet αSort u_4} (h : (a : α) → β (toUpperSet a)) (a : WithUpperSet α) :
            β a

            A recursor for WithUpperSet. Use as induction x.

            Equations
            Instances For
              theorem Topology.WithUpperSet.ofUpperSet_le_iff {α : Type u_1} [Preorder α] {a b : WithUpperSet α} :
              ofUpperSet a ofUpperSet b a b
              theorem Topology.WithUpperSet.toUpperSet_le_iff {α : Type u_1} [Preorder α] {a b : α} :
              toUpperSet a toUpperSet b a b
              def Topology.WithLowerSet (α : Type u_4) :
              Type u_4

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

              Equations
              Instances For
                @[match_pattern]

                toLowerSet is the identity function to the WithLowerSet of a type.

                Equations
                Instances For
                  @[match_pattern]

                  ofLowerSet is the identity function from the WithLowerSet of a type.

                  Equations
                  Instances For
                    @[deprecated Topology.WithLowerSet.toLowerSet_symm (since := "2024-10-10")]

                    Alias of Topology.WithLowerSet.toLowerSet_symm.

                    @[deprecated Topology.WithLowerSet.ofLowerSet_symm (since := "2024-10-10")]

                    Alias of Topology.WithLowerSet.ofLowerSet_symm.

                    @[simp]
                    theorem Topology.WithLowerSet.toLowerSet_ofLowerSet {α : Type u_1} (a : WithLowerSet α) :
                    toLowerSet (ofLowerSet a) = a
                    @[simp]
                    theorem Topology.WithLowerSet.ofLowerSet_toLowerSet {α : Type u_1} (a : α) :
                    ofLowerSet (toLowerSet a) = a
                    theorem Topology.WithLowerSet.toLowerSet_inj {α : Type u_1} {a b : α} :
                    toLowerSet a = toLowerSet b a = b
                    theorem Topology.WithLowerSet.ofLowerSet_inj {α : Type u_1} {a b : WithLowerSet α} :
                    ofLowerSet a = ofLowerSet b a = b
                    def Topology.WithLowerSet.rec {α : Type u_1} {β : WithLowerSet αSort u_4} (h : (a : α) → β (toLowerSet a)) (a : WithLowerSet α) :
                    β a

                    A recursor for WithLowerSet. Use as induction x.

                    Equations
                    Instances For
                      theorem Topology.WithLowerSet.ofLowerSet_le_iff {α : Type u_1} [Preorder α] {a b : WithLowerSet α} :
                      ofLowerSet a ofLowerSet b a b
                      theorem Topology.WithLowerSet.toLowerSet_le_iff {α : Type u_1} [Preorder α] {a b : α} :
                      toLowerSet a toLowerSet b a b

                      The Upper Set topology is homeomorphic to the Lower Set topology on the dual order

                      Equations
                      Instances For
                        class Topology.IsUpperSet (α : Type u_4) [t : TopologicalSpace α] [Preorder α] :

                        Prop-valued mixin for an ordered topological space to be The upper set topology is the topology where the open sets are the upper sets. In general the upper set topology does not coincide with the upper topology.

                        • topology_eq_upperSetTopology : t = upperSet α
                        Instances
                          class Topology.IsLowerSet (α : Type u_4) [t : TopologicalSpace α] [Preorder α] :

                          The lower set topology is the topology where the open sets are the lower sets. In general the lower set topology does not coincide with the lower topology.

                          • topology_eq_lowerSetTopology : t = lowerSet α
                          Instances

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

                            Equations
                            Instances For
                              @[simp]

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

                              theorem Topology.IsUpperSet.upperSet_le_upper {α : Type u_1} [Preorder α] {t₁ t₂ : TopologicalSpace α} [Topology.IsUpperSet α] [IsUpper α] :
                              t₁ t₂

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

                              Equations
                              Instances For
                                @[simp]

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

                                theorem Topology.IsLowerSet.lowerSet_le_lower {α : Type u_1} [Preorder α] {t₁ t₂ : TopologicalSpace α} [Topology.IsLowerSet α] [IsLower α] :
                                t₁ t₂
                                def Topology.WithUpperSet.map {α : Type u_1} {β : Type u_2} [Preorder α] [Preorder β] (f : α →o β) :

                                A monotone map between preorders spaces induces a continuous map between themselves considered with the upper set topology.

                                Equations
                                Instances For
                                  @[simp]
                                  theorem Topology.WithUpperSet.map_comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [Preorder α] [Preorder β] [Preorder γ] (g : β →o γ) (f : α →o β) :
                                  map (g.comp f) = (map g).comp (map f)
                                  @[simp]
                                  theorem Topology.WithUpperSet.toUpperSet_specializes_toUpperSet {α : Type u_1} [Preorder α] {a b : α} :
                                  toUpperSet a toUpperSet b b a
                                  @[simp]
                                  theorem Topology.WithUpperSet.ofUpperSet_le_ofUpperSet {α : Type u_1} [Preorder α] {a b : WithUpperSet α} :
                                  ofUpperSet a ofUpperSet b b a
                                  def Topology.WithLowerSet.map {α : Type u_1} {β : Type u_2} [Preorder α] [Preorder β] (f : α →o β) :

                                  A monotone map between preorders spaces induces a continuous map between themselves considered with the lower set topology.

                                  Equations
                                  Instances For
                                    @[simp]
                                    theorem Topology.WithLowerSet.map_comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [Preorder α] [Preorder β] [Preorder γ] (g : β →o γ) (f : α →o β) :
                                    map (g.comp f) = (map g).comp (map f)
                                    @[simp]
                                    theorem Topology.WithLowerSet.toLowerSet_specializes_toLowerSet {α : Type u_1} [Preorder α] {a b : α} :
                                    toLowerSet a toLowerSet b a b
                                    @[simp]
                                    theorem Topology.WithLowerSet.ofLowerSet_le_ofLowerSet {α : Type u_1} [Preorder α] {a b : WithLowerSet α} :
                                    ofLowerSet a ofLowerSet b a b