Crash.agda 279 B

1234567891011121314151617181920212223
  1. module Crash where
  2. data Nat : Set where
  3. zero : Nat
  4. suc : Nat -> Nat
  5. data Bool : Set where
  6. true : Bool
  7. false : Bool
  8. F : Bool -> Set
  9. F true = Nat
  10. F false = Bool
  11. not : Bool -> Bool
  12. not true = false
  13. not false = true
  14. h : ((x : F ?) -> F (not x)) -> Nat
  15. h g = g zero