diff 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
line wrap: on
line diff
--- a/agda/basic.agda	Tue Oct 07 14:55:40 2014 +0900
+++ b/agda/basic.agda	Tue Oct 07 15:09:17 2014 +0900
@@ -1,10 +1,12 @@
+open import Level
+
 module basic where
 
-id : {A : Set} -> A -> A
+id : {l : Level} {A : Set} -> A -> A
 id x = x
 
-_∙_ : {A B C : Set} -> (A -> B) -> (B -> C) -> (A -> C)
-f ∙ g = \x -> g (f x)
+_∙_ : {l ll lll : Level} {A : Set l} {B : Set ll} {C : Set lll} -> (B -> C) -> (A -> B) -> (A -> C)
+f ∙ g = \x -> f (g x)
 
 postulate String : Set
 postulate show   : {A : Set} -> A -> String
\ No newline at end of file