Category of categories #
This file contains the definition of the category Cat of all categories.
In this category objects are categories and
morphisms are functors between these categories.
Implementation notes #
Though Cat is not a concrete category, we use bundled to define
its carrier type.
Category of categories.
Instances For
Equations
- CategoryTheory.Cat.instInhabited = { default := { α := Type ?u.2, str := CategoryTheory.types } }
Equations
Equations
- CategoryTheory.Cat.instQuiver = { Hom := fun (C D : CategoryTheory.Cat) => C.Hom D }
The 1-morphism in Cat corresponding to a functor.
Instances For
The equivalence between the type of functors between two categories and the type of 1-morphisms in Cat between the objects corresponding to those categories.
Equations
- CategoryTheory.Functor.equivCatHom C D = { toFun := CategoryTheory.Functor.toCatHom, invFun := CategoryTheory.Cat.Hom.toFunctor, left_inv := ⋯, right_inv := ⋯ }
Instances For
The equivalence between the type of 1-morphisms in Cat between two objects and the type of functors between the categories corresponding to those objects.
Equations
Instances For
Equations
- CategoryTheory.Cat.Hom.instQuiver = { Hom := fun (F G : C ⟶ D) => CategoryTheory.Cat.Hom₂ F G }
The 2-morphism in Cat corresponding to a natural transformation between functors.
Equations
- CategoryTheory.NatTrans.toCatHom₂ η = { toNatTrans := η }
Instances For
Equations
- One or more equations did not get rendered due to their size.
The 2-iso in Cat corresponding to a natural isomorphism.
Equations
- CategoryTheory.Cat.Hom.isoMk e = { hom := CategoryTheory.NatTrans.toCatHom₂ e.hom, inv := CategoryTheory.NatTrans.toCatHom₂ e.inv, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The natural isomorphism corresponding to a 2-iso in Cat
Equations
- CategoryTheory.Cat.Hom.toNatIso e = { hom := e.hom.toNatTrans, inv := e.inv.toNatTrans, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Bicategory structure on Cat
Equations
- One or more equations did not get rendered due to their size.
Cat is a strict bicategory.
Category structure on Cat
The identity in the category of categories equals the identity functor.
Functor that gets the set of objects of a category. It is not
called forget, because it is not a faithful functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
See through the defeq objects.obj X = X.
Equations
Under certain hypotheses, an equivalence of categories actually
defines an isomorphism in Cat.