Built with Alectryon, running Coq+SerAPI v8.18.0+0.18.3. Bubbles () indicate interactive fragments: hover for details, tap to reveal contents. Use Ctrl+↑ Ctrl+↓ to navigate, Ctrl+🖱️ to focus. On Mac, use instead of Ctrl.
[Loading ML file number_string_notation_plugin.cmxs (using legacy method) ... done]
Require Import WildCat.Core. (** Unit category *)

IsGraph Unit

IsGraph Unit

Unit -> Unit -> Type
intros; exact Unit. Defined.

Is01Cat Unit

Is01Cat Unit

forall a : Unit, a $-> a

forall a b c : Unit, (b $-> c) -> (a $-> b) -> a $-> c
all: intros; exact tt. Defined.

Is0Gpd Unit

Is0Gpd Unit
constructor; intros; exact tt. Defined. Global Instance is2graph_unit : Is2Graph Unit := fun f g => isgraph_unit.

Is1Cat Unit

Is1Cat Unit

forall (a b c : Unit) (g : b $-> c), Is0Functor (cat_postcomp a g)

forall (a b c : Unit) (f : a $-> b), Is0Functor (cat_precomp c f)

forall (a b c d : Unit) (f : a $-> b) (g : b $-> c) (h : c $-> d), h $o g $o f $== h $o (g $o f)

forall (a b c d : Unit) (f : a $-> b) (g : b $-> c) (h : c $-> d), h $o (g $o f) $== h $o g $o f

forall (a b : Unit) (f : a $-> b), Id b $o f $== f

forall (a b : Unit) (f : a $-> b), f $o Id a $== f
a, b, c: Unit
g: b $-> c

forall a0 b0 : a $-> b, (a0 $-> b0) -> cat_postcomp a g a0 $-> cat_postcomp a g b0
a, b, c: Unit
f: a $-> b
forall a0 b0 : b $-> c, (a0 $-> b0) -> cat_precomp c f a0 $-> cat_precomp c f b0

forall (a b c d : Unit) (f : a $-> b) (g : b $-> c) (h : c $-> d), h $o g $o f $== h $o (g $o f)

forall (a b c d : Unit) (f : a $-> b) (g : b $-> c) (h : c $-> d), h $o (g $o f) $== h $o g $o f

forall (a b : Unit) (f : a $-> b), Id b $o f $== f

forall (a b : Unit) (f : a $-> b), f $o Id a $== f
all:intros; exact tt. Defined.