The dualizing functor on Cat
#
We define a (strict) functor opFunctor
and an equivalence assigning opposite categories to
categories. We then show that this functor is strictly involutive and that it induces an
equivalence on Cat
.
The endofunctor Cat ⥤ Cat
assigning to each category its opposite category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural isomorphism between the double application of Cat.opFunctor
and the
identity functor on Cat
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
The equivalence Cat ≌ Cat
associating each category with its opposite category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
CategoryTheory.Cat.opEquivalence_counitIso :
opEquivalence.counitIso = NatIso.ofComponents
(fun (x : Cat) => { hom := unopUnop ↑x, inv := opOp ↑((Functor.id Cat).obj x), hom_inv_id := ⋯, inv_hom_id := ⋯ })
@opEquivalence.proof_6
@[simp]
theorem
CategoryTheory.Cat.opEquivalence_unitIso :
opEquivalence.unitIso = NatIso.ofComponents
(fun (x : Cat) => { hom := opOp ↑((Functor.id Cat).obj x), inv := unopUnop ↑x, hom_inv_id := ⋯, inv_hom_id := ⋯ })
@opEquivalence.proof_3