Bool.agda 176 B

1234567891011
  1. module Bool where
  2. data Bool : Set where
  3. true : Bool
  4. false : Bool
  5. if_then_else_ : {A : Set} -> Bool -> A -> A -> A
  6. if true then x else y = x
  7. if false then x else y = y