view systemT/systemT.agda @ 3:36c9175d9adb

Migrate moggi from atton/agda/moggi (0:530373ccbcee)
author Yasutaka Higa <e115763@ie.u-ryukyu.ac.jp>
date Sun, 02 Nov 2014 09:41:29 +0900
parents fe247f476ecb
children
line wrap: on
line source

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