Idris2Doc : Data.String.Iterator

Data.String.Iterator

Reexports

importpublic Data.List.Lazy

Definitions

dataStringIterator : String->Type
Totality: total
Visibility: export
withString : (str : String) -> ((1_ : StringIteratorstr) ->a) ->a
Totality: total
Visibility: export
withIteratorString : (str : String) -> (1_ : StringIteratorstr) -> (String->a) ->a
  Runs the action `f` on the slice `res` of the original string `str` represented by the
iterator `it`
dataUnconsResult : String->Type
Totality: total
Visibility: public export
Constructors:
EOF : UnconsResultstr
Character : Char-> (1_ : StringIteratorstr) ->UnconsResultstr
uncons : (str : String) -> (1_ : StringIteratorstr) ->UnconsResultstr
foldl : (accTy->Char->accTy) ->accTy->String->accTy
Totality: total
Visibility: export
unpack : String->LazyListChar
Totality: total
Visibility: export