Library HoTT.Categories.Functor.Identity

Identity functor

Require Import Category.Core Functor.Core.

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

Section identity.
There is an identity functor. It does the obvious thing.
  Definition identity C : Functor C C
    := Build_Functor C C
                     (fun xx)
                     (fun _ _ xx)
                     (fun _ _ _ _ _idpath)
                     (fun _idpath).
End identity.

Module Export FunctorIdentityNotations.
  Notation "1" := (identity _) : functor_scope.
End FunctorIdentityNotations.