Skip to content

Instantly share code, notes, and snippets.

@jcommelin
Last active September 6, 2022 08:18
Show Gist options
  • Save jcommelin/82fb937a00b064f763d6a4644caa9403 to your computer and use it in GitHub Desktop.
Save jcommelin/82fb937a00b064f763d6a4644caa9403 to your computer and use it in GitHub Desktop.
Yoneda template
import category_theory.yoneda
import tactic.apply_fun
.
open category_theory opposite
/-! # Yoneda -/
variables (C : Type) [category.{0} C]
-- how to define a natural transformation
def nat_trans_hint (F : C ⥤ C) :
F ⟶ F :=
{ app := _ }
@[simps]
def yoneda : C ⥤ (Cᵒᵖ ⥤ Type) :=
{ obj := _,
map := _ }
.
lemma yoneda_faithful :
faithful (yoneda C) :=
begin
sorry
end
def yoneda_full :
full (yoneda C) :=
begin
sorry
end
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment