aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-29 13:49:09 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-29 13:49:09 +0000
commit27b1061be797da05212500f16af9c88ac28849ee (patch)
treef5520299455df7cef91c795aa07aaae90ec2d7ae /theories/Bool
parent32a24e55a8e38cd5db37224575269eb4355fdb30 (diff)
ajout option , Exc --> option, et lemmes dans les theories
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1914 85f007b7-540e-0410-9357-904b9bb8a0f7
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 *)