aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/Sumbool.v
diff options
context:
space:
mode:
authorGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-09 07:59:19 +0000
committerGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-09 07:59:19 +0000
commitdf9a4f1ae642cbbd2a6f1a3b82ad8169b7ec5ae6 (patch)
tree47f00369a7e6ceef22bdd4ab7406091b58108924 /theories/Bool/Sumbool.v
parentc04fe01b5d33b5e091c8fd19047514a7e4c4f311 (diff)
Making the sumbool functions transparent, so that they can used to
compute even inside Coq. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2846 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/Sumbool.v')
-rw-r--r--theories/Bool/Sumbool.v24
1 files changed, 12 insertions, 12 deletions
diff --git a/theories/Bool/Sumbool.v b/theories/Bool/Sumbool.v
index 84e74f86b..6f3adcf32 100644
--- a/theories/Bool/Sumbool.v
+++ b/theories/Bool/Sumbool.v
@@ -15,22 +15,22 @@
(** A boolean is either [true] or [false], and this is decidable *)
-Lemma sumbool_of_bool : (b:bool) {b=true}+{b=false}.
+Definition sumbool_of_bool : (b:bool) {b=true}+{b=false}.
Proof.
Induction b; Auto.
-Qed.
+Defined.
Hints Resolve sumbool_of_bool : bool.
-Lemma bool_eq_rec : (b:bool)(P:bool->Set)
+Definition bool_eq_rec : (b:bool)(P:bool->Set)
((b=true)->(P true))->((b=false)->(P false))->(P b).
Induction b; Auto.
-Qed.
+Defined.
-Lemma bool_eq_ind : (b:bool)(P:bool->Prop)
+Definition bool_eq_ind : (b:bool)(P:bool->Prop)
((b=true)->(P true))->((b=false)->(P false))->(P b).
Induction b; Auto.
-Qed.
+Defined.
(*i pourquoi ce machin-la est dans BOOL et pas dans LOGIC ? Papageno i*)
@@ -44,20 +44,20 @@ Variables A,B,C,D : Prop.
Hypothesis H1 : {A}+{B}.
Hypothesis H2 : {C}+{D}.
-Lemma sumbool_and : {A/\C}+{B\/D}.
+Definition sumbool_and : {A/\C}+{B\/D}.
Proof.
Case H1; Case H2; Auto.
-Qed.
+Defined.
-Lemma sumbool_or : {A\/C}+{B/\D}.
+Definition sumbool_or : {A\/C}+{B/\D}.
Proof.
Case H1; Case H2; Auto.
-Qed.
+Defined.
-Lemma sumbool_not : {B}+{A}.
+Definition sumbool_not : {B}+{A}.
Proof.
Case H1; Auto.
-Qed.
+Defined.
End connectives.