Skip to content

Commit

Permalink
Update Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Joël Riou <[email protected]>
  • Loading branch information
emilyriehl and joelriou authored Feb 25, 2025
1 parent 14a1fbd commit d90e5fe
Showing 1 changed file with 1 addition and 1 deletion.
Original file line number Diff line number Diff line change
Expand Up @@ -77,7 +77,7 @@ theorem nerve₂Adj.counit.naturality {C D : Type u} [SmallCategory C] [SmallCat
ReflQuiv.adj.counit).naturality _

/-- The counit of `nerve₂Adj.` -/
def nerve₂Adj.counit : nerveFunctor₂ ⋙ hoFunctor₂.{u} ⟶ (𝟭 Cat) where
def nerve₂Adj.counit : nerveFunctor₂ ⋙ hoFunctor₂.{u} ⟶ 𝟭 Cat where
app C := nerve₂Adj.counit.app (Cat.of C)
naturality _ _ F := nerve₂Adj.counit.naturality F

Expand Down

0 comments on commit d90e5fe

Please sign in to comment.