Idris2Doc : Data.Linear.Communications

Data.Linear.Communications(source)

This module is based on the content of the functional pearl
How to Take the Inverse of a Type
by Daniel Marshall and Dominic Orchard

Definitions

dataProtocol : Type
Totality: total
Visibility: public export
Constructors:
Send : Type->Protocol->Protocol
Recv : Type->Protocol->Protocol
End : Protocol
Dual : Protocol->Protocol
Totality: total
Visibility: public export
dataLChan : Protocol->Type
Totality: total
Visibility: export
Constructor: 
MkLChan : LChanp