Library HoTT.Categories.NaturalTransformation.Composition.Functorial

Functoriality of composition of natural transformations

Require Import Category.Core Functor.Core.
Require Import FunctorCategory.Core Functor.Composition.Core NaturalTransformation.Composition.Core NaturalTransformation.Composition.Laws.

Set Universe Polymorphism.
Set Implicit Arguments.
Generalizable All Variables.
Set Asymmetric Patterns.

Local Open Scope functor_scope.

Section functorial_composition.
  Context `{Funext}.
  Variables C D E : PreCategory.

  Local Open Scope natural_transformation_scope.

whiskering on the left is a functor

  Definition whiskerL_functor (F : (D E)%category)
  : ((C D) (C E))%category
    := Build_Functor
         (C D) (C E)
         (fun GF o G)%functor
         (fun _ _ TF oL T)
         (fun _ _ _ _ _composition_of_whisker_l _ _ _)
         (fun _whisker_l_right_identity _ _).

whiskering on the right is a functor

  Definition whiskerR_functor (G : (C D)%category)
  : ((D E) (C E))%category
    := Build_Functor
         (D E) (C E)
         (fun FF o G)%functor
         (fun _ _ TT oR G)
         (fun _ _ _ _ _composition_of_whisker_r _ _ _)
         (fun _whisker_r_left_identity _ _).
End functorial_composition.