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
  • Topology.upperSet α = { IsOpen := IsUpperSet, isOpen_univ := , isOpen_inter := , isOpen_sUnion := }
Instances For

    Topology whose open sets are lower sets.

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

    Equations
    • Topology.lowerSet α = { IsOpen := IsLowerSet, isOpen_univ := , isOpen_inter := , isOpen_sUnion := }
    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
            @[simp]
            theorem Topology.WithUpperSet.to_WithUpperSet_symm_eq {α : Type u_1} :
            Topology.WithUpperSet.toUpperSet.symm = Topology.WithUpperSet.ofUpperSet
            @[simp]
            theorem Topology.WithUpperSet.of_WithUpperSet_symm_eq {α : Type u_1} :
            Topology.WithUpperSet.ofUpperSet.symm = Topology.WithUpperSet.toUpperSet
            @[simp]
            theorem Topology.WithUpperSet.toUpperSet_ofUpperSet {α : Type u_1} (a : Topology.WithUpperSet α) :
            Topology.WithUpperSet.toUpperSet (Topology.WithUpperSet.ofUpperSet a) = a
            @[simp]
            theorem Topology.WithUpperSet.ofUpperSet_toUpperSet {α : Type u_1} (a : α) :
            Topology.WithUpperSet.ofUpperSet (Topology.WithUpperSet.toUpperSet a) = a
            theorem Topology.WithUpperSet.toUpperSet_inj {α : Type u_1} {a : α} {b : α} :
            Topology.WithUpperSet.toUpperSet a = Topology.WithUpperSet.toUpperSet b a = b
            theorem Topology.WithUpperSet.ofUpperSet_inj {α : Type u_1} {a : Topology.WithUpperSet α} {b : Topology.WithUpperSet α} :
            Topology.WithUpperSet.ofUpperSet a = Topology.WithUpperSet.ofUpperSet b a = b
            def Topology.WithUpperSet.rec {α : Type u_1} {β : Topology.WithUpperSet αSort u_4} (h : (a : α) → β (Topology.WithUpperSet.toUpperSet a)) (a : Topology.WithUpperSet α) :
            β a

            A recursor for WithUpperSet. Use as induction x using WithUpperSet.rec.

            Equations
            Instances For
              Equations
              • Topology.WithUpperSet.instInhabitedWithUpperSet = inst
              Equations
              • Topology.WithUpperSet.instPreorderWithUpperSet = inst
              Equations
              theorem Topology.WithUpperSet.ofUpperSet_le_iff {α : Type u_1} [Preorder α] {a : Topology.WithUpperSet α} {b : Topology.WithUpperSet α} :
              Topology.WithUpperSet.ofUpperSet a Topology.WithUpperSet.ofUpperSet b a b
              theorem Topology.WithUpperSet.toUpperSet_le_iff {α : Type u_1} [Preorder α] {a : α} {b : α} :
              Topology.WithUpperSet.toUpperSet a Topology.WithUpperSet.toUpperSet b a b

              ofUpperSet as an OrderIso

              Equations
              • Topology.WithUpperSet.ofUpperSetOrderIso = { toEquiv := Topology.WithUpperSet.ofUpperSet, map_rel_iff' := }
              Instances For

                toUpperSet as an OrderIso

                Equations
                • Topology.WithUpperSet.toUpperSetOrderIso = { toEquiv := Topology.WithUpperSet.toUpperSet, map_rel_iff' := }
                Instances For
                  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
                        @[simp]
                        theorem Topology.WithLowerSet.to_WithLowerSet_symm_eq {α : Type u_1} :
                        Topology.WithLowerSet.toLowerSet.symm = Topology.WithLowerSet.ofLowerSet
                        @[simp]
                        theorem Topology.WithLowerSet.of_WithLowerSet_symm_eq {α : Type u_1} :
                        Topology.WithLowerSet.ofLowerSet.symm = Topology.WithLowerSet.toLowerSet
                        @[simp]
                        theorem Topology.WithLowerSet.toLowerSet_ofLowerSet {α : Type u_1} (a : Topology.WithLowerSet α) :
                        Topology.WithLowerSet.toLowerSet (Topology.WithLowerSet.ofLowerSet a) = a
                        @[simp]
                        theorem Topology.WithLowerSet.ofLowerSet_toLowerSet {α : Type u_1} (a : α) :
                        Topology.WithLowerSet.ofLowerSet (Topology.WithLowerSet.toLowerSet a) = a
                        theorem Topology.WithLowerSet.toLowerSet_inj {α : Type u_1} {a : α} {b : α} :
                        Topology.WithLowerSet.toLowerSet a = Topology.WithLowerSet.toLowerSet b a = b
                        theorem Topology.WithLowerSet.ofLowerSet_inj {α : Type u_1} {a : Topology.WithLowerSet α} {b : Topology.WithLowerSet α} :
                        Topology.WithLowerSet.ofLowerSet a = Topology.WithLowerSet.ofLowerSet b a = b
                        def Topology.WithLowerSet.rec {α : Type u_1} {β : Topology.WithLowerSet αSort u_4} (h : (a : α) → β (Topology.WithLowerSet.toLowerSet a)) (a : Topology.WithLowerSet α) :
                        β a

                        A recursor for WithLowerSet. Use as induction x using WithLowerSet.rec.

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

                          ofLowerSet as an OrderIso

                          Equations
                          • Topology.WithLowerSet.ofLowerSetOrderIso = { toEquiv := Topology.WithLowerSet.ofLowerSet, map_rel_iff' := }
                          Instances For

                            toLowerSet as an OrderIso

                            Equations
                            • Topology.WithLowerSet.toLowerSetOrderIso = { toEquiv := Topology.WithLowerSet.toLowerSet, map_rel_iff' := }
                            Instances For

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

                              Equations
                              • Topology.WithUpperSet.toDualHomeomorph = { toEquiv := { toFun := OrderDual.toDual, invFun := OrderDual.ofDual, left_inv := , right_inv := }, continuous_toFun := , continuous_invFun := }
                              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.

                                Instances
                                  Equations
                                  • =
                                  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.

                                  Instances
                                    Equations
                                    • =

                                    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].

                                      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].

                                        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.toUpperSet_specializes_toUpperSet {α : Type u_1} [Preorder α] {a : α} {b : α} :
                                          Topology.WithUpperSet.toUpperSet a Topology.WithUpperSet.toUpperSet b b a
                                          @[simp]
                                          theorem Topology.WithUpperSet.ofUpperSet_le_ofUpperSet {α : Type u_1} [Preorder α] {a : Topology.WithUpperSet α} {b : Topology.WithUpperSet α} :
                                          Topology.WithUpperSet.ofUpperSet a Topology.WithUpperSet.ofUpperSet b b a
                                          @[simp]
                                          theorem Topology.WithUpperSet.isUpperSet_toUpperSet_preimage {α : Type u_1} [Preorder α] {s : Set (Topology.WithUpperSet α)} :
                                          IsUpperSet (Topology.WithUpperSet.toUpperSet ⁻¹' s) IsOpen s
                                          @[simp]
                                          theorem Topology.WithUpperSet.isOpen_ofUpperSet_preimage {α : Type u_1} [Preorder α] {s : Set α} :
                                          IsOpen (Topology.WithUpperSet.ofUpperSet ⁻¹' s) IsUpperSet s

                                          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.toLowerSet_specializes_toLowerSet {α : Type u_1} [Preorder α] {a : α} {b : α} :
                                            Topology.WithLowerSet.toLowerSet a Topology.WithLowerSet.toLowerSet b a b
                                            @[simp]
                                            theorem Topology.WithLowerSet.ofLowerSet_le_ofLowerSet {α : Type u_1} [Preorder α] {a : Topology.WithLowerSet α} {b : Topology.WithLowerSet α} :
                                            Topology.WithLowerSet.ofLowerSet a Topology.WithLowerSet.ofLowerSet b a b
                                            @[simp]
                                            theorem Topology.WithLowerSet.isLowerSet_toLowerSet_preimage {α : Type u_1} [Preorder α] {s : Set (Topology.WithLowerSet α)} :
                                            IsLowerSet (Topology.WithLowerSet.toLowerSet ⁻¹' s) IsOpen s
                                            @[simp]
                                            theorem Topology.WithLowerSet.isOpen_ofLowerSet_preimage {α : Type u_1} [Preorder α] {s : Set α} :
                                            IsOpen (Topology.WithLowerSet.ofLowerSet ⁻¹' s) IsLowerSet s