aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-28 14:08:18 +0000
committerGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-28 14:08:18 +0000
commit4800380437b6b133c7a9346aafa9c4e2b76527d7 (patch)
tree447b2dfbd93d1e12dc7dcf47f5fd8f105d8d09a1 /theories/Bool
parent4c36f26e02e8c1df3f0851250526d89fd81d8448 (diff)
Elimination du '
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1000 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index c49c4bf8e..f546a1aa1 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -221,12 +221,12 @@ Save.
Lemma orb_prop :
(a,b:bool)(orb a b)=true -> (a = true)\/(b = true).
-Induction a; Induction b; Simpl; Try '(Intro H;Discriminate H); Auto with bool.
+Induction a; Induction b; Simpl; Try (Intro H;Discriminate H); Auto with bool.
Save.
Lemma orb_prop2 :
(a,b:bool)(Is_true (orb a b)) -> (Is_true a)\/(Is_true b).
-Induction a; Induction b; Simpl; Try '(Intro H;Discriminate H); Auto with bool.
+Induction a; Induction b; Simpl; Try (Intro H;Discriminate H); Auto with bool.
Save.
Lemma orb_true_intro
@@ -304,7 +304,7 @@ Lemma andb_prop :
(a,b:bool)(andb a b) = true -> (a = true)/\(b = true).
Proof.
- Induction a; Induction b; Simpl; Try '(Intro H;Discriminate H);
+ Induction a; Induction b; Simpl; Try (Intro H;Discriminate H);
Auto with bool.
Save.
Hints Resolve andb_prop : bool v62.
@@ -312,7 +312,7 @@ Hints Resolve andb_prop : bool v62.
Lemma andb_prop2 :
(a,b:bool)(Is_true (andb a b)) -> (Is_true a)/\(Is_true b).
Proof.
- Induction a; Induction b; Simpl; Try '(Intro H;Discriminate H);
+ Induction a; Induction b; Simpl; Try (Intro H;Discriminate H);
Auto with bool.
Save.
Hints Resolve andb_prop2 : bool v62.