Skip to content

Commit

Permalink
chore(CategoryTheory/DiscreteCategory): remove unecessary line in pro…
Browse files Browse the repository at this point in the history
…of (#12382)
  • Loading branch information
callesonne committed Apr 23, 2024
1 parent ec75ee1 commit f0ba14a
Showing 1 changed file with 0 additions and 1 deletion.
1 change: 0 additions & 1 deletion Mathlib/CategoryTheory/DiscreteCategory.lean
Expand Up @@ -54,7 +54,6 @@ structure Discrete (α : Type u₁) where

@[simp]
theorem Discrete.mk_as {α : Type u₁} (X : Discrete α) : Discrete.mk X.as = X := by
ext
rfl
#align category_theory.discrete.mk_as CategoryTheory.Discrete.mk_as

Expand Down

0 comments on commit f0ba14a

Please sign in to comment.