Idris2Doc : Data.List.Lazy.Quantifiers

Data.List.Lazy.Quantifiers

WIP: same as Data.List.Quantifiers but for lazy lists

Definitions

dataAny : (a->Type) ->LazyLista->Type
Totality: total
Visibility: public export
Constructors:
Here : px->Anyp (x::xs)
There : Anyp (Force xs) ->Anyp (x::xs)
toExists : Anypxs->Existsp
Totality: total
Visibility: public export
toDPair : Anypxs->DPairap
Totality: total
Visibility: public export