comparison agda/basic.agda @ 35:c5cdbedc68ad

Proof Monad-law-2-2
author Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp>
date Sat, 18 Oct 2014 14:15:13 +0900
parents e0ba1bf564dd
children 743c05b98dad
comparison
equal deleted inserted replaced
34:b7c4e6276bcf 35:c5cdbedc68ad
1 open import Level 1 open import Level
2 2
3 module basic where 3 module basic where
4 4
5 id : {l : Level} {A : Set} -> A -> A 5 id : {l : Level} {A : Set l} -> A -> A
6 id x = x 6 id x = x
7 7
8 _∙_ : {l ll lll : Level} {A : Set l} {B : Set ll} {C : Set lll} -> (B -> C) -> (A -> B) -> (A -> C) 8 _∙_ : {l ll lll : Level} {A : Set l} {B : Set ll} {C : Set lll} -> (B -> C) -> (A -> B) -> (A -> C)
9 f ∙ g = \x -> f (g x) 9 f ∙ g = \x -> f (g x)
10 10