aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-27 14:20:23 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-27 14:20:23 +0000
commit8972b118c89d7840c13ead05d5e826667f66dc2a (patch)
tree59142ef989e383e28386e00ebc7dd343529f9ef0 /theories/Bool
parented97a490501de3693a8990b0f53deae43dba01a7 (diff)
Simplification de deux preuves. En outre ca simplifie leur extraction.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2082 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 3c82fd8e9..57c10f256 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -261,7 +261,7 @@ Trivial with bool.
Save.
Lemma orb_true_elim : (b1,b2:bool)(orb b1 b2)=true -> {b1=true}+{b2=true}.
-NewDestruct b1; [Auto with bool | NewDestruct b2; Auto with bool].
+NewDestruct b1; Simpl; Auto with bool.
Save.
Lemma orb_false_intro
: (b1,b2:bool)(b1=false)->(b2=false)->(orb b1 b2)=false.
@@ -371,7 +371,7 @@ Save.
Lemma andb_false_elim :
(b1,b2:bool)(andb b1 b2)=false -> {b1=false}+{b2=false}.
-NewDestruct b1; NewDestruct b2; Simpl; Auto with bool.
+NewDestruct b1; Simpl; Auto with bool.
Save.
Hints Resolve andb_false_elim : bool v62.