Skip to content

Commit

Permalink
Refactor(Mathlib/CategoryTheory/Core): Make functorToCore compute (#1…
Browse files Browse the repository at this point in the history
…0649)

Change `functorToCore` to use `Groupoid.inv` instead of `IsIso.inv` and as a consequence make it's computable.
  • Loading branch information
Shamrock-Frost committed Feb 18, 2024
1 parent a13e804 commit f6d4f4c
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Core.lean
Expand Up @@ -77,9 +77,9 @@ variable {C} {G : Type u₂} [Groupoid.{v₂} G]
-- Note that this function is not functorial
-- (consider the two functors from [0] to [1], and the natural transformation between them).
/-- A functor from a groupoid to a category C factors through the core of C. -/
noncomputable def functorToCore (F : G ⥤ C) : G ⥤ Core C where
def functorToCore (F : G ⥤ C) : G ⥤ Core C where
obj X := F.obj X
map f := ⟨F.map f, F.map (inv f), _, _⟩
map f := ⟨F.map f, F.map (Groupoid.inv f), _, _⟩
#align category_theory.core.functor_to_core CategoryTheory.Core.functorToCore

/-- We can functorially associate to any functor from a groupoid to the core of a category `C`,
Expand Down

0 comments on commit f6d4f4c

Please sign in to comment.