Skip to content

Commit

Permalink
feat(category_theory/const): Constant functor of object from punit
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Dec 3, 2018
1 parent 5856459 commit e507633
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions category_theory/const.lean
Expand Up @@ -4,6 +4,7 @@

import category_theory.functor_category
import category_theory.isomorphism
import category_theory.punit

universes u₁ v₁ u₂ v₂ u₃ v₃

Expand Down Expand Up @@ -47,4 +48,13 @@ include 𝒟

end

omit 𝒥
def of : C ⥤ (punit ⥤ C) := const punit

namespace of
@[simp] lemma obj_obj (X : C) : (of.obj X).obj = λ _, X := rfl
@[simp] lemma obj_map (X : C) : (of.obj X).map = λ _ _ _, 𝟙 X := rfl
@[simp] lemma map_app {X Y : C} (f : X ⟶ Y) : (of.map f).app = λ _, f := rfl
end of

end category_theory.functor

0 comments on commit e507633

Please sign in to comment.