aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Bool')
-rw-r--r--theories/Bool/Sumbool.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/theories/Bool/Sumbool.v b/theories/Bool/Sumbool.v
index 9c6cd1f42..275712084 100644
--- a/theories/Bool/Sumbool.v
+++ b/theories/Bool/Sumbool.v
@@ -23,6 +23,17 @@ Save.
Hints Resolve sumbool_of_bool : bool.
+Lemma bool_eq_rec : (b:bool)(P:bool->Set)
+ ((b=true)->(P true))->((b=false)->(P false))->(P b).
+Induction b; Auto.
+Save.
+
+Lemma bool_eq_ind : (b:bool)(P:bool->Prop)
+ ((b=true)->(P true))->((b=false)->(P false))->(P b).
+Induction b; Auto.
+Save.
+
+
(*i pourquoi ce machin-la est dans BOOL et pas dans LOGIC ? Papageno i*)
(* Logic connectives on type sumbool *)