Skip to content

Commit

Permalink
chore(CategoryTheory.ConcreteCategory): inline `ConcreteCategory.forg…
Browse files Browse the repository at this point in the history
…et` (#19217)

We already make `forget` `reducible` and further declarations downstream of it `abbrev`'s. It makes sense to `inline` it also to avoid Lean noticing it.
  • Loading branch information
mattrobball committed Nov 23, 2024
1 parent 8eedc61 commit ba61bf3
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/ConcreteCategory/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -55,7 +55,7 @@ class ConcreteCategory (C : Type u) [Category.{v} C] where
/-- That functor is faithful -/
[forget_faithful : forget.Faithful]

attribute [reducible] ConcreteCategory.forget
attribute [inline, reducible] ConcreteCategory.forget
attribute [instance] ConcreteCategory.forget_faithful

/-- The forgetful functor from a concrete category to `Type u`. -/
Expand Down

0 comments on commit ba61bf3

Please sign in to comment.