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 involving product categories *)
[Loading ML file number_string_notation_plugin.cmxs (using legacy method) ... done]
Require Import Types.Prod. Set Universe Polymorphism. Set Implicit Arguments. Generalizable All Variables. Set Asymmetric Patterns. (** ** Product of natural transformations *) Section prod. Context {A : PreCategory}. Context {B : PreCategory}. Context {C : PreCategory}. Variables F F' : Functor A B. Variables G G' : Functor A C. Variable T : NaturalTransformation F F'. Variable U : NaturalTransformation G G'. Definition prod : NaturalTransformation (F * G) (F' * G') := Build_NaturalTransformation (F * G) (F' * G') (fun x : A => (T x, U x)) (fun _ _ _ => path_prod' (commutes T _ _ _) (commutes U _ _ _)). End prod. Local Infix "*" := prod : natural_transformation_scope. (** ** Natural transformations between partially applied functors *) Section induced. Variables C D E : PreCategory. Variable F : Functor (C * D) E. Local Ltac t := simpl; intros; rewrite <- !composition_of; simpl; rewrite ?left_identity, ?right_identity; reflexivity.
C, D, E: PreCategory
F: Functor (C * D) E
s, d: C
m: morphism C s d

NaturalTransformation (induced_snd F s) (induced_snd F d)
C, D, E: PreCategory
F: Functor (C * D) E
s, d: C
m: morphism C s d

NaturalTransformation (induced_snd F s) (induced_snd F d)
C, D, E: PreCategory
F: Functor (C * D) E
s, d: C
m: morphism C s d

forall (s0 d0 : D) (m0 : morphism D s0 d0), (F _1 (m, 1) o (induced_snd F s) _1 m0)%morphism = ((induced_snd F d) _1 m0 o F _1 (m, 1))%morphism
abstract t. Defined.
C, D, E: PreCategory
F: Functor (C * D) E
s, d: D
m: morphism D s d

NaturalTransformation (Core.induced_fst F s) (Core.induced_fst F d)
C, D, E: PreCategory
F: Functor (C * D) E
s, d: D
m: morphism D s d

NaturalTransformation (Core.induced_fst F s) (Core.induced_fst F d)
C, D, E: PreCategory
F: Functor (C * D) E
s, d: D
m: morphism D s d

forall (s0 d0 : C) (m0 : morphism C s0 d0), (F _1 (1, m) o (Core.induced_fst F s) _1 m0)%morphism = ((Core.induced_fst F d) _1 m0 o F _1 (1, m))%morphism
abstract t. Defined. End induced. Module Export NaturalTransformationProdNotations. Infix "*" := prod : natural_transformation_scope. End NaturalTransformationProdNotations.