Representatives of small categories #
Given a type Ω : Type w
, we construct a structure SmallCategoryOfSet Ω : Type w
which consists of the data and axioms that allows to define a category
structure such that the type of objects and morphisms identify to subtypes of Ω
.
This allows to define a small family of small categories
SmallCategoryOfSet.categoryFamily : SmallCategoryOfSet Ω → Type w
which, up to equivalence, represents all categories such that
types of objects and morphisms have cardinalities less than or equal to
that of Ω
(see SmallCategoryOfSet.exists_equivalence
).
Structure which allows to construct a category whose types
of objects and morphisms are subtypes of a fixed type Ω
.
- obj : Set Ω
objects
morphisms
identity morphisms
the composition of morphisms
Instances For
Equations
- One or more equations did not get rendered due to their size.
The family of all categories such that the types of objects and
morphisms are subtypes of a given type Ω
.
Equations
Instances For
Helper structure for the construction of a term in SmallCategoryOfSet
.
This involves the choice of bijections between types of objects and morphisms
in a category C
and subtypes of a type Ω
.
- obj : Set Ω
objects
morphisms
a bijection between the types of objects
a bijection between the types of morphisms
Instances For
The SmallCategoryOfSet
structure induced by a
CoreSmallCategoryOfSet
structure.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given h : CoreSmallCategoryOfSet Ω C
, this is the
obvious functor h.smallCategoryOfSet.obj ⥤ C
.
Equations
Instances For
Given h : CoreSmallCategoryOfSet Ω C
,
the obvious functor h.smallCategoryOfSet.obj ⥤ C
is fully faithful.
Equations
- h.fullyFaithfulFunctor = { preimage := fun {X Y : ↑h.smallCategoryOfSet.obj} => ⇑h.homEquiv.symm, map_preimage := ⋯, preimage_map := ⋯ }
Instances For
Given h : CoreSmallCategoryOfSet Ω C
,
the obvious functor h.smallCategoryOfSet.obj ⥤ C
is an equivalence.