diff systemT/systemT.agda @ 1:fe247f476ecb

Migrate systemT from atton/agda/systemT (13:5a81867278af)
author Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp>
date Sun, 02 Nov 2014 09:40:54 +0900
parents
children
line wrap: on
line diff
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/systemT/systemT.agda	Sun Nov 02 09:40:54 2014 +0900
@@ -0,0 +1,17 @@
+module systemT where
+
+data Bool : Set where
+  T : Bool
+  F : Bool
+
+data Int : Set where
+  O : Int
+  S : Int -> Int
+
+R : {U : Set} -> U -> (U -> (Int -> U)) -> Int -> U
+R u v O = u
+R u v (S t) = v (R u v t) t
+
+D : {U : Set} -> U -> U -> Bool -> U
+D u v F = v
+D u v T = u
\ No newline at end of file