Skip to content

Commit a49be33

Browse files
committed
fixes after rebase
1 parent ec6ca92 commit a49be33

File tree

2 files changed

+6
-6
lines changed

2 files changed

+6
-6
lines changed

src/Std/Data/DHashMap/Internal/AssocList/Iterator.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -32,8 +32,8 @@ public instance : Iterator (α := AssocListIterator α β) Id ((a : α) × β a)
3232
| .skip _ => False
3333
| .done => it.internalState.l = .nil
3434
step it := pure (match it with
35-
| ⟨⟨.nil⟩⟩ => ⟨.done, rfl⟩
36-
| ⟨⟨.cons k v l⟩⟩ => ⟨.yield (toIterM ⟨l⟩ Id _) ⟨k, v⟩, rfl⟩)
35+
| ⟨⟨.nil⟩⟩ => .deflate ⟨.done, rfl⟩
36+
| ⟨⟨.cons k v l⟩⟩ => .deflate ⟨.yield (toIterM ⟨l⟩ Id _) ⟨k, v⟩, rfl⟩)
3737

3838
def AssocListIterator.finitenessRelation :
3939
FinitenessRelation (AssocListIterator α β) Id where

src/Std/Data/DHashMap/IteratorLemmas.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -22,13 +22,13 @@ open Std.Iterators
2222

2323
@[simp]
2424
public theorem step_iter_nil {α : Type u} {β : α → Type v} :
25-
((.nil : AssocList α β).iter).step = ⟨.done, rfl⟩ :=
26-
(rfl)
25+
((.nil : AssocList α β).iter).step = ⟨.done, rfl⟩ := by
26+
simp [Iter.step, IterM.step, Iterator.step, Iter.toIterM, iter]
2727

2828
@[simp]
2929
public theorem step_iter_cons {α : Type u} {β : α → Type v} {k v} {l : AssocList α β} :
30-
((AssocList.cons k v l).iter).step = ⟨.yield l.iter ⟨k, v⟩, rfl⟩ :=
31-
(rfl)
30+
((AssocList.cons k v l).iter).step = ⟨.yield l.iter ⟨k, v⟩, rfl⟩ := by
31+
simp [Iter.step, IterM.step, Iterator.step, Iter.toIterM, iter, toIterM, IterM.toIter]
3232

3333
@[simp]
3434
public theorem toList_iter {α : Type u} {β : α → Type v} {l : AssocList α β} :

0 commit comments

Comments
 (0)