Basics on the category of relations #
We define the category of types CategoryTheory.RelCat
with binary relations as morphisms.
Associating each function with the relation defined by its graph yields a faithful and
essentially surjective functor graphFunctor
that also characterizes all isomorphisms
(see rel_iso_iff
).
By flipping the arguments to a relation, we construct an equivalence opEquivalence
between
RelCat
and its opposite.
A type synonym for Type u
, which carries the category instance for which
morphisms are binary relations.
Equations
- CategoryTheory.RelCat = Type ?u.3
Instances For
The category of types with binary relations as morphisms.
theorem
CategoryTheory.RelCat.Hom.rel_comp_apply₂
{X Y Z : RelCat}
(f : X ⟶ Y)
(g : Y ⟶ Z)
(x : X)
(z : Z)
:
The essentially surjective faithful embedding from the category of types and functions into the category of types and relations.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
@[simp]
@[simp]