instance
String.Slice.Pattern.instInhabitedForwardCharPredSearcher
{a✝ : Char → Bool}
{a✝¹ : Slice}
:
Inhabited (ForwardCharPredSearcher a✝ a✝¹)
def
String.Slice.Pattern.instInhabitedForwardCharPredSearcher.default
{a✝ : Char → Bool}
{a✝¹ : Slice}
:
ForwardCharPredSearcher a✝ a✝¹
Equations
Instances For
@[inline]
def
String.Slice.Pattern.ForwardCharPredSearcher.iter
(p : Char → Bool)
(s : Slice)
:
Std.Iter (SearchStep s)
Equations
Instances For
instance
String.Slice.Pattern.ForwardCharPredSearcher.instIteratorIdSearchStep
{p : Char → Bool}
(s : Slice)
:
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.
Instances For
instance
String.Slice.Pattern.ForwardCharPredSearcher.instFiniteIdSearchStep
{p : Char → Bool}
{s : Slice}
:
instance
String.Slice.Pattern.ForwardCharPredSearcher.instIteratorLoopIdSearchStep
{p : Char → Bool}
{s : Slice}
:
@[defaultInstance 1000]
instance
String.Slice.Pattern.ForwardCharPredSearcher.instToForwardSearcherForallCharPropDecide
{p : Char → Prop}
[DecidablePred p]
:
ToForwardSearcher p (ForwardCharPredSearcher fun (b : Char) => decide (p b))
Equations
- String.Slice.Pattern.ForwardCharPredSearcher.instToForwardSearcherForallCharPropDecide = { toSearcher := String.Slice.Pattern.ForwardCharPredSearcher.iter fun (x : Char) => decide (p x) }
Equations
Instances For
@[inline]
def
String.Slice.Pattern.BackwardCharPredSearcher.iter
(c : Char → Bool)
(s : Slice)
:
Std.Iter (SearchStep s)
Equations
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.
Instances For
@[defaultInstance 1000]
@[defaultInstance 1000]
instance
String.Slice.Pattern.BackwardCharPredSearcher.instToBackwardSearcherForallCharPropOfDecidablePred
{p : Char → Prop}
[DecidablePred p]
:
Equations
- One or more equations did not get rendered due to their size.