Idris2Doc : Data.Vect.Binary

Data.Vect.Binary(source)

The content of this file is taken from the paper
Heterogeneous Binary Random-access lists

Definitions

dataBVect : Nat->Bin->Type->Type
Totality: total
Visibility: public export
Constructors:
Nil : BVectn [] a
(::) : IMaybe (isIb) (Treena) ->BVect (Sn) bsa->BVectn (b::bs) a
dataPath : Nat->Bin->Type
Totality: total
Visibility: public export
Constructors:
Here : Pathn->Pathn (I::bs)
There : Path (Sn) bs->Pathn (b::bs)
zero : Pathn (sucbs)
Totality: total
Visibility: public export
lookup : BVectnbsa->Pathnbs->a
Totality: total
Visibility: public export
cons : Treena->BVectnbsa->BVectn (sucbs) a
Totality: total
Visibility: public export