Proj.agda 352 B

123456789101112131415161718192021
  1. module Proj where
  2. open import AlonzoPrelude
  3. showTrue : True -> String
  4. showTrue _ = "tt"
  5. -- data True : Set where
  6. -- tt : True
  7. data T4 : Set where
  8. C : True -> True -> True -> True -> T4
  9. g : True -> True -> True
  10. g x y = tt
  11. f14 : T4 -> True -> True
  12. f14 (C x y z t) = \w -> g x t
  13. mainS : String
  14. mainS = showTrue $ (id ○ f14) (C tt tt tt tt) tt