Documentation

Mathlib.Topology.Category.TopCat.Opens

The category of open sets in a topological space. #

We define toTopCat : Opens X ⥤ TopCat and map (f : X ⟶ Y) : Opens Y ⥤ Opens X, given by taking preimages of open sets.

Unfortunately Opens isn't (usefully) a functor TopCat ⥤ Cat. (One can in fact define such a functor, but using it results in unresolvable Eq.rec terms in goals.)

Really it's a 2-functor from (spaces, continuous functions, equalities) to (categories, functors, natural isomorphisms). We don't attempt to set up the full theory here, but do provide the natural isomorphisms mapId : map (𝟙 X) ≅ 𝟭 (opens X) and mapComp : map (f ≫ g) ≅ map g ⋙ map f.

Beyond that, there's a collection of simp lemmas for working with these constructions.

Since Opens X has a partial order, it automatically receives a Category instance. Unfortunately, because we do not allow morphisms in Prop, the morphisms U ⟶ V are not just proofs U ≤ V, but rather ULift (PLift (U ≤ V)).

instance TopologicalSpace.Opens.opensHomHasCoeToFun {X : TopCat} {U : TopologicalSpace.Opens X} {V : TopologicalSpace.Opens X} :
CoeFun (U V) fun (x : U V) => UV
Equations
  • TopologicalSpace.Opens.opensHomHasCoeToFun = { coe := fun (f : U V) (x : U) => { val := x, property := } }

We now construct as morphisms various inclusions of open sets.

The inclusion U ⊓ V ⟶ U as a morphism in the category of open sets.

Equations
Instances For

    The inclusion U ⊓ V ⟶ V as a morphism in the category of open sets.

    Equations
    Instances For
      noncomputable def TopologicalSpace.Opens.leSupr {X : TopCat} {ι : Type u_1} (U : ιTopologicalSpace.Opens X) (i : ι) :
      U i iSup U

      The inclusion U i ⟶ supr U as a morphism in the category of open sets.

      Equations
      Instances For
        noncomputable def TopologicalSpace.Opens.botLE {X : TopCat} (U : TopologicalSpace.Opens X) :

        The inclusion ⊥ ⟶ U as a morphism in the category of open sets.

        Equations
        Instances For
          noncomputable def TopologicalSpace.Opens.leTop {X : TopCat} (U : TopologicalSpace.Opens X) :

          The inclusion U ⟶ ⊤ as a morphism in the category of open sets.

          Equations
          Instances For
            theorem TopologicalSpace.Opens.infLELeft_apply {X : TopCat} (U : TopologicalSpace.Opens X) (V : TopologicalSpace.Opens X) (x : (U V)) :
            (fun (x : (U V)) => { val := x, property := }) x = { val := x, property := }
            @[simp]
            theorem TopologicalSpace.Opens.infLELeft_apply_mk {X : TopCat} (U : TopologicalSpace.Opens X) (V : TopologicalSpace.Opens X) (x : X) (m : x U V) :
            (fun (x : (U V)) => { val := x, property := }) { val := x, property := m } = { val := x, property := }
            @[simp]
            theorem TopologicalSpace.Opens.leSupr_apply_mk {X : TopCat} {ι : Type u_1} (U : ιTopologicalSpace.Opens X) (i : ι) (x : X) (m : x U i) :
            (fun (x : (U i)) => { val := x, property := }) { val := x, property := m } = { val := x, property := }

            The functor from open sets in X to Top, realising each open set as a topological space itself.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              theorem TopologicalSpace.Opens.toTopCat_map (X : TopCat) {U : TopologicalSpace.Opens X} {V : TopologicalSpace.Opens X} {f : U V} {x : X} {h : x U} :
              ((TopologicalSpace.Opens.toTopCat X).map f) { val := x, property := h } = { val := x, property := }

              The inclusion map from an open subset to the whole space, as a morphism in TopCat.

              Equations
              Instances For

                The inclusion of the top open subset (i.e. the whole space) is an isomorphism.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For

                  Opens.map f gives the functor from open sets in Y to open set in X, given by taking preimages under f.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    @[simp]
                    theorem TopologicalSpace.Opens.map_coe {X : TopCat} {Y : TopCat} (f : X Y) (U : TopologicalSpace.Opens Y) :
                    ((TopologicalSpace.Opens.map f).obj U) = f ⁻¹' U
                    @[simp]
                    theorem TopologicalSpace.Opens.map_obj {X : TopCat} {Y : TopCat} (f : X Y) (U : Set Y) (p : IsOpen U) :
                    (TopologicalSpace.Opens.map f).obj { carrier := U, is_open' := p } = { carrier := f ⁻¹' U, is_open' := }
                    @[simp]
                    theorem TopologicalSpace.Opens.map_id_obj' {X : TopCat} (U : Set X) (p : IsOpen U) :
                    (TopologicalSpace.Opens.map (CategoryTheory.CategoryStruct.id X)).obj { carrier := U, is_open' := p } = { carrier := U, is_open' := p }
                    noncomputable def TopologicalSpace.Opens.leMapTop {X : TopCat} {Y : TopCat} (f : X Y) (U : TopologicalSpace.Opens X) :

                    The inclusion U ⟶ (map f).obj ⊤ as a morphism in the category of open sets.

                    Equations
                    Instances For
                      @[simp]
                      theorem TopologicalSpace.Opens.map_comp_obj' {X : TopCat} {Y : TopCat} {Z : TopCat} (f : X Y) (g : Y Z) (U : Set Z) (p : IsOpen U) :
                      (TopologicalSpace.Opens.map (CategoryTheory.CategoryStruct.comp f g)).obj { carrier := U, is_open' := p } = (TopologicalSpace.Opens.map f).obj ((TopologicalSpace.Opens.map g).obj { carrier := U, is_open' := p })
                      theorem TopologicalSpace.Opens.map_iSup {X : TopCat} {Y : TopCat} (f : X Y) {ι : Type u_1} (U : ιTopologicalSpace.Opens Y) :

                      The functor Opens X ⥤ Opens X given by taking preimages under the identity function is naturally isomorphic to the identity functor.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For

                        The natural isomorphism between taking preimages under f ≫ g, and the composite of taking preimages under g, then preimages under f.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For

                          If two continuous maps f g : X ⟶ Y are equal, then the functors Opens Y ⥤ Opens X they induce are isomorphic.

                          Equations
                          Instances For
                            @[simp]
                            theorem TopologicalSpace.Opens.mapIso_hom_app {X : TopCat} {Y : TopCat} (f : X Y) (g : X Y) (h : f = g) (U : TopologicalSpace.Opens Y) :
                            @[simp]
                            theorem TopologicalSpace.Opens.mapIso_inv_app {X : TopCat} {Y : TopCat} (f : X Y) (g : X Y) (h : f = g) (U : TopologicalSpace.Opens Y) :

                            A homeomorphism of spaces gives an equivalence of categories of open sets.

                            TODO: define OrderIso.equivalence, use it.

                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              @[simp]
                              theorem IsOpenMap.functor_obj_coe {X : TopCat} {Y : TopCat} {f : X Y} (hf : IsOpenMap f) (U : TopologicalSpace.Opens X) :
                              ((IsOpenMap.functor hf).obj U) = f '' U

                              An open map f : X ⟶ Y induces a functor Opens X ⥤ Opens Y.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For

                                An open map f : X ⟶ Y induces an adjunction between Opens X and Opens Y.

                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Equations
                                  • =