File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed
Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -19,7 +19,7 @@ open Std.Iterators Std.PRange
1919
2020namespace Std.Slice.List
2121
22- theorem internalIter_rco_eq {α : Type u} {s : ListSlice α} :
22+ theorem internalIter_eq {α : Type u} {s : ListSlice α} :
2323 Internal.iter s = match s.internalRepresentation.stop with
2424 | some stop => s.internalRepresentation.list.iter.take stop
2525 | none => s.internalRepresentation.list.iter.toTake := by
@@ -29,7 +29,7 @@ theorem toList_internalIter {α : Type u} {s : ListSlice α} :
2929 (Internal.iter s).toList = match s.internalRepresentation.stop with
3030 | some stop => s.internalRepresentation.list.take stop
3131 | none => s.internalRepresentation.list := by
32- simp only [internalIter_rco_eq ]
32+ simp only [internalIter_eq ]
3333 split <;> simp
3434
3535theorem internalIter_eq_toIteratorIter {α : Type u} {s : ListSlice α} :
You can’t perform that action at this time.
0 commit comments