RTN.agda 109 B

12345678
  1. module RTN where
  2. data Nat : Set where
  3. zero : Nat
  4. suc : Nat -> Nat
  5. {-# BUILTIN NATURAL Nat #-}