Idris2Doc : Data.Zippable

Data.Zippable

Definitions

interfaceZippable : (Type->Type) ->Type
  The `Zippable` interface describes how you can combine and split the
elements in a parameterised type.
@ z the parameterised type

Parameters: z
Methods:
zipWith : (a->b->c) ->za->zb->zc
  Combine two parameterised types by applying a function.
@ z the parameterised type
@ func the function to combine elements with
zip : za->zb->z (a, b)
  Combine two parameterised types into a parameterised type of pairs.
@ z the parameterised type

Fixity Declaration: infixr operator, level 6
zipWith3 : (a->b->c->d) ->za->zb->zc->zd
  Combine three parameterised types by applying a function.
@ z the parameterised type
@ func the function to combine elements with
zip3 : za->zb->zc->z (a, (b, c))
  Combine three parameterised types into a parameterised type of triplets.
@ z the parameterised type
unzipWith : (a-> (b, c)) ->za-> (zb, zc)
  Split a parameterised type by applying a function into a pair of
parameterised types.
@ z the parameterised type
@ func the function to split elements with
unzip : z (a, b) -> (za, zb)
  Split a parameterised type of pairs into a pair of parameterised types.
@ z the parameterised type
unzipWith3 : (a-> (b, (c, d))) ->za-> (zb, (zc, zd))
  Split a parameterised type by applying a function into a triplet of
parameterised types.
@ z the parameterised type
@ func the function to split elements with
unzip3 : z (a, (b, c)) -> (za, (zb, zc))
  Split a parameterised type of triplets into a triplet of parameterised
types.
@ z the parameterised type

Implementations:
Zippable (Vectk)
ZippableStream
ZippableColist1
ZippableColist
ZippableList
ZippableList1
zipWith : Zippablez=> (a->b->c) ->za->zb->zc
  Combine two parameterised types by applying a function.
@ z the parameterised type
@ func the function to combine elements with

Totality: total
Visibility: public export
zip : Zippablez=>za->zb->z (a, b)
  Combine two parameterised types into a parameterised type of pairs.
@ z the parameterised type

Totality: total
Visibility: public export
Fixity Declaration: infixr operator, level 6
zipWith3 : Zippablez=> (a->b->c->d) ->za->zb->zc->zd
  Combine three parameterised types by applying a function.
@ z the parameterised type
@ func the function to combine elements with

Totality: total
Visibility: public export
zip3 : Zippablez=>za->zb->zc->z (a, (b, c))
  Combine three parameterised types into a parameterised type of triplets.
@ z the parameterised type

Totality: total
Visibility: public export
unzipWith : Zippablez=> (a-> (b, c)) ->za-> (zb, zc)
  Split a parameterised type by applying a function into a pair of
parameterised types.
@ z the parameterised type
@ func the function to split elements with

Totality: total
Visibility: public export
unzip : Zippablez=>z (a, b) -> (za, zb)
  Split a parameterised type of pairs into a pair of parameterised types.
@ z the parameterised type

Totality: total
Visibility: public export
unzipWith3 : Zippablez=> (a-> (b, (c, d))) ->za-> (zb, (zc, zd))
  Split a parameterised type by applying a function into a triplet of
parameterised types.
@ z the parameterised type
@ func the function to split elements with

Totality: total
Visibility: public export
unzip3 : Zippablez=>z (a, (b, c)) -> (za, (zb, zc))
  Split a parameterised type of triplets into a triplet of parameterised
types.
@ z the parameterised type

Totality: total
Visibility: public export