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 d90e5fe commit 5556a3a
Showing 1 changed file with 1 addition and 1 deletion.
Original file line number Diff line number Diff line change
Expand Up @@ -251,7 +251,7 @@ theorem toNerve₂.mk_naturality : toNerve₂.mk.naturalityProperty F = ⊤ :=
recovered from the underlying ReflPrefunctor. -/
@[simps!]
def toNerve₂.mk : X ⟶ nerveFunctor₂.obj (Cat.of C) where
app := fun n => toNerve₂.mk.app F n.unop
app n := toNerve₂.mk.app F n.unop
naturality _ _ f := MorphismProperty.of_eq_top (toNerve₂.mk_naturality F hyp) f.unop

end
Expand Down

0 comments on commit 5556a3a

Please sign in to comment.