Mercurial > hg > Members > atton > delta_monad
view agda/basic.agda @ 31:33b386de3f56
Proof list-associative
author | Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp> |
---|---|
date | Sat, 18 Oct 2014 13:38:29 +0900 |
parents | e0ba1bf564dd |
children | c5cdbedc68ad |
line wrap: on
line source
open import Level module basic where id : {l : Level} {A : Set} -> A -> A id x = 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