2 ||M|| This file is part of HELM, an Hypertextual, Electronic
3 ||A|| Library of Mathematics, developed at the Computer Science
4 ||T|| Department of the University of Bologna, Italy.
8 \ / This file is distributed under the terms of the
9 \ / GNU General Public License Version 2
10 V_______________________________________________________________ *)
12 include "basics/relations.ma".
14 (********** bool **********)
15 inductive bool: Type[0] ≝
19 (* destruct does not work *)
20 theorem not_eq_true_false : true ≠ false.
21 @nmk #Heq change with match true with [true ⇒ False|false ⇒ True]
24 definition notb : bool → bool ≝
25 λ b:bool. match b with [true ⇒ false|false ⇒ true ].
27 interpretation "boolean not" 'not x = (notb x).
29 theorem notb_elim: ∀ b:bool.∀ P:bool → Prop.
32 | false ⇒ P true] → P (notb b).
33 #b #P elim b normalize // qed.
35 theorem notb_notb: ∀b:bool. notb (notb b) = b.
38 theorem injective_notb: injective bool bool notb.
41 definition andb : bool → bool → bool ≝
42 λb1,b2:bool. match b1 with [ true ⇒ b2 | false ⇒ false ].
44 interpretation "boolean and" 'and x y = (andb x y).
46 theorem andb_elim: ∀ b1,b2:bool. ∀ P:bool → Prop.
47 match b1 with [ true ⇒ P b2 | false ⇒ P false] → P (b1 ∧ b2).
48 #b1 #b2 #P (elim b1) normalize // qed.
50 theorem andb_true_l: ∀ b1,b2. (b1 ∧ b2) = true → b1 = true.
51 #b1 (cases b1) normalize // qed.
53 theorem andb_true_r: ∀b1,b2. (b1 ∧ b2) = true → b2 = true.
54 #b1 #b2 (cases b1) normalize // (cases b2) // qed.
56 definition orb : bool → bool → bool ≝
57 λb1,b2:bool.match b1 with [ true ⇒ true | false ⇒ b2].
59 interpretation "boolean or" 'or x y = (orb x y).
61 theorem orb_elim: ∀ b1,b2:bool. ∀ P:bool → Prop.
62 match b1 with [ true ⇒ P true | false ⇒ P b2] → P (orb b1 b2).
63 #b1 #b2 #P (elim b1) normalize // qed.
65 definition if_then_else: ∀A:Type[0]. bool → A → A → A ≝
66 λA.λb.λ P,Q:A. match b with [ true ⇒ P | false ⇒ Q].
68 theorem bool_to_decidable_eq:
69 ∀b1,b2:bool. decidable (b1=b2).
70 #b1 #b2 (cases b1) (cases b2) /2/ %2 /3/ qed.
72 theorem true_or_false:
73 ∀b:bool. b = true ∨ b = false.