- empty {s : Slice} (pos : s.Pos) : ForwardSliceSearcher s
- proper {s : Slice} (needle : Slice) (table : Array Pos.Raw) (stackPos needlePos : Pos.Raw) : ForwardSliceSearcher s
- atEnd {s : Slice} : ForwardSliceSearcher s
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
@[irreducible]
def
String.Slice.Pattern.ForwardSliceSearcher.instIteratorIdSearchStep.findNext
(s needle : Slice)
(table : Array Pos.Raw)
(stackPos needlePos startPos currStackPos needlePos✝ : Pos.Raw)
(h : stackPos ≤ currStackPos)
:
Id
(Std.Shrink
(Std.Iterators.PlausibleIterStep fun (x : Std.Iterators.IterStep (Std.IterM Id (SearchStep s)) (SearchStep s)) =>
match x with
| Std.Iterators.IterStep.yield it' out =>
match { internalState := proper needle table stackPos needlePos }.internalState with
| empty pos => (∃ (newPos : s.Pos), pos < newPos ∧ it'.internalState = empty newPos) ∨ it'.internalState = atEnd
| proper needle table stackPos needlePos =>
(∃ (newStackPos : Pos.Raw), ∃ (newNeedlePos : Pos.Raw), stackPos < newStackPos ∧ newStackPos ≤ s.rawEndPos ∧ it'.internalState = proper needle table newStackPos newNeedlePos) ∨ it'.internalState = atEnd
| atEnd => False
| Std.Iterators.IterStep.skip it => False
| Std.Iterators.IterStep.done => True))
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.