view agda/basic.agda @ 145:b93e4b2aea9e

Add prototype Delta for modification with type changes
author Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp>
date Fri, 27 Feb 2015 14:49:55 +0900
parents 55d11ce7e223
children
line wrap: on
line source

open import Level

module basic where

id : {l : Level} {A : Set l} -> A -> A
id x = x

_∙_ : {l : Level} {A B C : Set l} -> (B -> C) -> (A -> B) -> (A -> C)
f ∙ g = \x -> f (g x)

postulate String : Set
postulate show   : {l : Level} {A : Set l} -> A -> String