Skip to content

Commit

Permalink
minor fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
mattrobball committed Feb 15, 2023
1 parent 8a683dd commit dadd6da
Showing 1 changed file with 7 additions and 7 deletions.
14 changes: 7 additions & 7 deletions Mathlib/CategoryTheory/Yoneda.lean
Original file line number Diff line number Diff line change
Expand Up @@ -31,7 +31,7 @@ open Opposite

universe v₁ u₁ u₂

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
variable {C : Type u₁} [Category.{v₁} C]

/-- The Yoneda embedding, as a functor from `C` into presheaves on `C`.
Expand All @@ -48,9 +48,9 @@ def yoneda : C ⥤ Cᵒᵖ ⥤ Type v₁
map_id := fun Y => by funext; dsimp; erw [Category.id_comp] }
map f :=
{ app := fun Y g => g ≫ f
naturality := sorry }
naturality := fun Y Y' g => by funext Z; aesop_cat }
map_id := by aesop_cat
map_comp := sorry
map_comp := fun f g => by ext Y; dsimp; funext f; simp
#align category_theory.yoneda CategoryTheory.yoneda

/-- The co-Yoneda embedding, as a functor from `Cᵒᵖ` into co-presheaves on `C`.
Expand All @@ -61,11 +61,11 @@ def coyoneda : Cᵒᵖ ⥤ C ⥤ Type v₁
obj X :=
{ obj := fun Y => unop X ⟶ Y
map := fun f g => g ≫ f
map_comp := sorry
map_id := sorry }
map_comp := fun f g => by funext; dsimp; erw [Category.assoc]
map_id := fun Y => by funext; dsimp; erw [Category.comp_id] }
map f :=
{ app := fun Y g => f.unop ≫ g
naturality := sorry }
naturality := fun Y Y' g => by funext Z; aesop_cat }
#align category_theory.coyoneda CategoryTheory.coyoneda

namespace Yoneda
Expand All @@ -88,7 +88,7 @@ See <https://stacks.math.columbia.edu/tag/001P>.
-/
instance yonedaFull : Full (yoneda : C ⥤ Cᵒᵖ ⥤ Type v₁) where
preimage {X} {Y} f := f.app (op X) (𝟙 X)
witness := sorry
witness {X} {Y} f := by dsimp; sorry
#align category_theory.yoneda.yoneda_full CategoryTheory.Yoneda.yonedaFull

/-- The Yoneda embedding is faithful.
Expand Down

0 comments on commit dadd6da

Please sign in to comment.