Skip to content

Commit 0061230

Browse files
committed
chore(Combinatorics/SetFamily/KruskalKatona): remove outdated comment (#30564)
The referenced diamond was fixed in #29436.
1 parent 0b502d5 commit 0061230

File tree

1 file changed

+0
-5
lines changed

1 file changed

+0
-5
lines changed

Mathlib/Combinatorics/SetFamily/KruskalKatona.lean

Lines changed: 0 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -42,11 +42,6 @@ The key results proved here are:
4242
kruskal-katona, kruskal, katona, shadow, initial segments, intersecting
4343
-/
4444

45-
-- TODO: There's currently a diamond. See https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/DecidableEq.20diamond.20on.20Fin
46-
-- import Mathlib.Order.Fin.Basic
47-
-- example (n : ℕ) : instDecidableEqFin n = instDecidableEq_mathlib := rfl
48-
attribute [-instance] instDecidableEqFin
49-
5045
open Nat
5146
open scoped FinsetFamily
5247

0 commit comments

Comments
 (0)