comparison agda/basic.agda @ 29:e0ba1bf564dd

Apply level to some functions
author Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp>
date Tue, 07 Oct 2014 15:09:17 +0900
parents 6e6d646d7722
children c5cdbedc68ad
comparison
equal deleted inserted replaced
28:6e6d646d7722 29:e0ba1bf564dd
1 open import Level
2
1 module basic where 3 module basic where
2 4
3 id : {A : Set} -> A -> A 5 id : {l : Level} {A : Set} -> A -> A
4 id x = x 6 id x = x
5 7
6 _∙_ : {A B C : Set} -> (A -> B) -> (B -> C) -> (A -> C) 8 _∙_ : {l ll lll : Level} {A : Set l} {B : Set ll} {C : Set lll} -> (B -> C) -> (A -> B) -> (A -> C)
7 f ∙ g = \x -> g (f x) 9 f ∙ g = \x -> f (g x)
8 10
9 postulate String : Set 11 postulate String : Set
10 postulate show : {A : Set} -> A -> String 12 postulate show : {A : Set} -> A -> String