comparison 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
comparison
equal deleted inserted replaced
27:742e62fc63e4 28:6e6d646d7722
1 module basic where
2
3 id : {A : Set} -> A -> A
4 id x = x
5
6 _∙_ : {A B C : Set} -> (A -> B) -> (B -> C) -> (A -> C)
7 f ∙ g = \x -> g (f x)
8
9 postulate String : Set
10 postulate show : {A : Set} -> A -> String