Mercurial > hg > Members > atton > delta_monad
view agda/basic.agda @ 28:6e6d646d7722
Split basic functions to file
author | Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp> |
---|---|
date | Tue, 07 Oct 2014 14:55:40 +0900 |
parents | |
children | e0ba1bf564dd |
line wrap: on
line source
module basic where id : {A : Set} -> A -> A id x = x _∙_ : {A B C : Set} -> (A -> B) -> (B -> C) -> (A -> C) f ∙ g = \x -> g (f x) postulate String : Set postulate show : {A : Set} -> A -> String