aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/Bool.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-04 13:29:45 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-03-04 13:29:45 +0000
commit6274447373e7dc69234da3415f8d9c4d4b67ced2 (patch)
treec2190c4f3ee24b87e49cec5927d02a77272ba42e /theories/Bool/Bool.v
parent9935f0d7ab63d31f7a4a8c05d90627dff41dabf8 (diff)
Nouveau Rewrite-in plus economique
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2507 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/Bool.v')
-rwxr-xr-xtheories/Bool/Bool.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index f8b50e6c2..1942ca6b3 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -449,7 +449,7 @@ Qed.
Lemma xorb_move_l_r_2 : (b,b',b'':bool) (xorb b b')=b'' -> b=(xorb b'' b').
Proof.
- Intros. Rewrite (xorb_comm b b') in H. Rewrite (xorb_move_l_r_1 b' b b'' H). Apply xorb_comm.
+ Intros. Rewrite xorb_comm in H. Rewrite (xorb_move_l_r_1 b' b b'' H). Apply xorb_comm.
Qed.
Lemma xorb_move_r_l_1 : (b,b',b'':bool) b=(xorb b' b'') -> (xorb b' b)=b''.