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.
(** * Natural transformations between functors from initial categories and to terminal categories *)
[Loading ML file number_string_notation_plugin.cmxs (using legacy method) ... done]
Require Import InitialTerminalCategory.Core InitialTerminalCategory.Functors. Require Import Contractible. Set Universe Polymorphism. Set Implicit Arguments. Generalizable All Variables. Set Asymmetric Patterns. Section NaturalTransformations. Variable C : PreCategory. Definition from_initial `{@IsInitialCategory zero} (F G : Functor zero C) : NaturalTransformation F G := Build_NaturalTransformation F G (fun x => initial_category_ind _ x) (fun x _ _ => initial_category_ind _ x).
C: PreCategory
H: Funext
zero: PreCategory
H0: IsInitialCategory zero
F, G: Functor zero C

Contr (NaturalTransformation F G)
C: PreCategory
H: Funext
zero: PreCategory
H0: IsInitialCategory zero
F, G: Functor zero C

Contr (NaturalTransformation F G)
C: PreCategory
H: Funext
zero: PreCategory
H0: IsInitialCategory zero
F, G: Functor zero C

forall y : NaturalTransformation F G, from_initial F G = y
abstract ( intros; apply path_natural_transformation; intro x; exact (initial_category_ind _ x) ). Defined. Local Existing Instance Functors.to_initial_category_empty. Global Instance trunc_to_initial `{Funext} `{@IsInitialCategory zero} (F G : Functor zero C) : Contr (NaturalTransformation F G) := trunc_from_initial F G. Definition to_terminal `{@IsTerminalCategory one H1 H2} (F G : Functor C one) : NaturalTransformation F G := Build_NaturalTransformation F G (fun x => center _) (fun _ _ _ => path_contr _ _).
C: PreCategory
H: Funext
one: PreCategory
H1: Contr one
H2: forall s d : one, Contr (morphism one s d)
H0: IsTerminalCategory one
F, G: Functor C one

Contr (NaturalTransformation F G)
C: PreCategory
H: Funext
one: PreCategory
H1: Contr one
H2: forall s d : one, Contr (morphism one s d)
H0: IsTerminalCategory one
F, G: Functor C one

Contr (NaturalTransformation F G)
C: PreCategory
H: Funext
one: PreCategory
H1: Contr one
H2: forall s d : one, Contr (morphism one s d)
H0: IsTerminalCategory one
F, G: Functor C one

forall y : NaturalTransformation F G, to_terminal F G = y
abstract (path_natural_transformation; exact (contr _)). Defined. End NaturalTransformations.