Sums and products of discrete categories. #
This file shows that binary products and binary sums of discrete categories
are also discrete, both in the form of explicit equivalences and through the
IsDiscrete
typeclass.
Main declarations #
Discrete.productEquiv
: The equivalence of categories betweenDiscrete (J × K)
andDiscrete J × Discrete K
Discrete.sumEquiv
: The equivalence of categories betweenDiscrete (J ⊕ K)
andDiscrete J ⊕ Discrete K
.IsDiscrete.prod
: anIsDiscrete
instance on the product of two discrete categories.IsDiscrete.sum
: anIsDiscrete
instance on the sum of two discrete categories.
instance
CategoryTheory.IsDiscrete.prod
(C : Type u_1)
[Category.{u_4, u_1} C]
(D : Type u_3)
[Category.{u_5, u_3} D]
[IsDiscrete C]
[IsDiscrete D]
:
IsDiscrete (C × D)
A product of discrete categories is discrete.
instance
CategoryTheory.IsDiscrete.sum
(C : Type u_1)
(C' : Type u_2)
[Category.{u_4, u_1} C]
[Category.{u_5, u_2} C']
[IsDiscrete C]
[IsDiscrete C']
:
IsDiscrete (C ⊕ C')
A product of discrete categories is discrete.