Skip to content

Commit fa0a740

Browse files
committed
remove todos
1 parent fc721a6 commit fa0a740

File tree

1 file changed

+0
-2
lines changed

1 file changed

+0
-2
lines changed

src/Init/Data/Iterators/Basic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -480,7 +480,6 @@ def IterM.TerminationMeasures.Finite.Rel
480480
instance {α : Type w} {m : Type w → Type w'} {β : Type w} [Iterator α m β]
481481
[Finite α m] : WellFoundedRelation (IterM.TerminationMeasures.Finite α m) where
482482
rel := IterM.TerminationMeasures.Finite.Rel
483-
-- TODO: workaround for module system issue?
484483
wf := by exact (InvImage.wf _ Finite.wf).transGen
485484

486485
/--
@@ -588,7 +587,6 @@ def IterM.TerminationMeasures.Productive.Rel
588587
instance {α : Type w} {m : Type w → Type w'} {β : Type w} [Iterator α m β]
589588
[Productive α m] : WellFoundedRelation (IterM.TerminationMeasures.Productive α m) where
590589
rel := IterM.TerminationMeasures.Productive.Rel
591-
-- TODO: workaround for module system issue?
592590
wf := by exact (InvImage.wf _ Productive.wf).transGen
593591

594592
/--

0 commit comments

Comments
 (0)