Bool.agda 349 B

123456789101112131415161718
  1. {-# OPTIONS --without-K #-}
  2. module Common.Bool where
  3. open import Agda.Builtin.Bool public
  4. not : Bool -> Bool
  5. not true = false
  6. not false = true
  7. notnot : Bool -> Bool
  8. notnot true = not (not true)
  9. notnot false = not (not false)
  10. if_then_else_ : ∀ {a} {A : Set a} → Bool → A → A → A
  11. if true then t else f = t
  12. if false then t else f = f