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.
(** * Pointwise Natural Transformations *)
[Loading ML file number_string_notation_plugin.cmxs (using legacy method) ... done]
Require Import FunctorCategory.Core NaturalTransformation.Paths Functor.Composition.Core NaturalTransformation.Composition.Core. Require Import Functor.Pointwise.Core. Set Universe Polymorphism. Set Implicit Arguments. Generalizable All Variables. Set Asymmetric Patterns. (** Recall that a "pointwise" functor is a functor [Aᴮ → Cᴰ] induced by functors [D → B] and [A → C]. Given two functors [D → B] and a natural transformation between them, there is an induced natural transformation between the resulting functors between functor categories, and similarly for two functors [A → C]. In this file, we construct these natural transformations. They will be used to construct the pointwise induced adjunction [Fˣ ⊣ Gˣ] of an adjunction [F ⊣ G] for all categories [X]. *) Local Open Scope morphism_scope. Local Open Scope category_scope. Local Open Scope functor_scope. Local Open Scope natural_transformation_scope. Section pointwise. Context `{Funext}. Variables C D C' D' : PreCategory. Local Ltac t := path_natural_transformation; simpl; rewrite <- ?composition_of; try apply ap; first [ apply commutes | symmetry; apply commutes ]. (** ** [Tˣ] for a natural transformation [T : F → G] and a functor [x : C → D] *)
H: Funext
C, D, C', D': PreCategory
F, G: Functor C D
T: NaturalTransformation F G
F': Functor C' D'

NaturalTransformation (pointwise F F') (pointwise G F')
H: Funext
C, D, C', D': PreCategory
F, G: Functor C D
T: NaturalTransformation F G
F': Functor C' D'

NaturalTransformation (pointwise F F') (pointwise G F')
H: Funext
C, D, C', D': PreCategory
F, G: Functor C D
T: NaturalTransformation F G
F': Functor C' D'

forall (s d : (D -> C')%category) (m : morphism (D -> C') s d), (F' o d oL T o (pointwise F F') _1 m)%morphism = ((pointwise G F') _1 m o (F' o s oL T))%morphism
abstract t. Defined. (** ** [Fᵀ] for a natural transformation [T : F' → G'] and a functor [F : C → D] *)
H: Funext
C, D, C', D': PreCategory
F: Functor C D
F', G': Functor C' D'
T': NaturalTransformation F' G'

NaturalTransformation (pointwise F F') (pointwise F G')
H: Funext
C, D, C', D': PreCategory
F: Functor C D
F', G': Functor C' D'
T': NaturalTransformation F' G'

NaturalTransformation (pointwise F F') (pointwise F G')
H: Funext
C, D, C', D': PreCategory
F: Functor C D
F', G': Functor C' D'
T': NaturalTransformation F' G'

forall (s d : (D -> C')%category) (m : morphism (D -> C') s d), (T' oR d oR F o (pointwise F F') _1 m)%morphism = ((pointwise F G') _1 m o (T' oR s oR F))%morphism
abstract t. Defined. End pointwise.