Documentation

Mathlib.CategoryTheory.Category.Bipointed

The category of bipointed types #

This defines Bipointed, the category of bipointed types.

TODO #

Monoidal structure

structure Bipointed :
Type (u + 1)

The category of bipointed types.

  • X : Type u

    The underlying type of a bipointed type.

  • toProd : self.X × self.X

    The two points of a bipointed type, bundled together as a pair.

Instances For
    @[reducible, inline]
    abbrev Bipointed.of {X : Type u_1} (to_prod : X × X) :

    Turns a bipointing into a bipointed type.

    Equations
    Instances For
      theorem Bipointed.coe_of {X : Type u_1} (to_prod : X × X) :
      (of to_prod).X = X
      def Prod.Bipointed {X : Type u_1} (to_prod : X × X) :

      Alias of Bipointed.of.


      Turns a bipointing into a bipointed type.

      Equations
      Instances For
        structure Bipointed.Hom (X Y : Bipointed) :

        Morphisms in Bipointed.

        Instances For
          theorem Bipointed.Hom.ext {X Y : Bipointed} {x y : X.Hom Y} (toFun : x.toFun = y.toFun) :
          x = y

          The identity morphism of X : Bipointed.

          Equations
          Instances For
            @[simp]
            theorem Bipointed.Hom.id_toFun (X : Bipointed) (a : X.X) :
            def Bipointed.Hom.comp {X Y Z : Bipointed} (f : X.Hom Y) (g : Y.Hom Z) :
            X.Hom Z

            Composition of morphisms of Bipointed.

            Equations
            Instances For
              @[simp]
              theorem Bipointed.Hom.comp_toFun {X Y Z : Bipointed} (f : X.Hom Y) (g : Y.Hom Z) (a✝ : X.X) :
              (f.comp g).toFun a✝ = (g.toFun f.toFun) a✝
              @[reducible, inline]
              abbrev Bipointed.HomSubtype (X : Bipointed) (Y : Bipointed) :
              Type (max 0 u_1 u_2)

              The subtype of functions corresponding to the morphisms in Bipointed.

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

                Swaps the pointed elements of a bipointed type. Prod.swap as a functor.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[simp]
                  theorem Bipointed.swap_obj_X (X : Bipointed) :
                  (swap.obj X).X = X.X
                  @[simp]
                  theorem Bipointed.swap_map_toFun {X✝ Y✝ : Bipointed} (f : X✝ Y✝) (a✝ : X✝.X) :
                  (swap.map f).toFun a✝ = f.toFun a✝

                  The equivalence between Bipointed and itself induced by Prod.swap both ways.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    @[simp]
                    theorem Bipointed.swapEquiv_functor_map_toFun {X✝ Y✝ : Bipointed} (f : X✝ Y✝) (a✝ : X✝.X) :
                    (swapEquiv.functor.map f).toFun a✝ = f.toFun a✝
                    @[simp]
                    theorem Bipointed.swapEquiv_inverse_map_toFun {X✝ Y✝ : Bipointed} (f : X✝ Y✝) (a✝ : X✝.X) :
                    (swapEquiv.inverse.map f).toFun a✝ = f.toFun a✝

                    The forgetful functor from Bipointed to Pointed which forgets about the second point.

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

                      The forgetful functor from Bipointed to Pointed which forgets about the first point.

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

                        The functor from Pointed to Bipointed which bipoints the point.

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

                          The functor from Pointed to Bipointed which adds a second point.

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

                            The functor from Pointed to Bipointed which adds a first point.

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

                              BipointedToPointed_fst is inverse to PointedToBipointed.

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

                                BipointedToPointed_snd is inverse to PointedToBipointed.

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

                                  The free/forgetful adjunction between PointedToBipointed_fst and BipointedToPointed_fst.

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

                                    The free/forgetful adjunction between PointedToBipointed_snd and BipointedToPointed_snd.

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