aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zmisc.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 13:59:36 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 13:59:36 +0000
commit9e2ba1d42bfeff9aafc8384fb131330b725ce3be (patch)
tree5e4c6a613580cec0230ba83471686506352eaf1d /theories/ZArith/Zmisc.v
parent6fe9381c21e6700791318920afd656a22c6a32b5 (diff)
Concentration des notations officielles dans Init/Notations; restructuration de Init
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4050 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zmisc.v')
-rw-r--r--theories/ZArith/Zmisc.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zmisc.v b/theories/ZArith/Zmisc.v
index 8a7a1caa4..414a230f0 100644
--- a/theories/ZArith/Zmisc.v
+++ b/theories/ZArith/Zmisc.v
@@ -546,7 +546,7 @@ Qed.
Lemma Zgt_is_le_bool : (x,y:Z) (Zgt x y) <-> (Zle_bool y `x-1`)=true.
Proof.
- Intros. Apply iff_trans with b:=`y < x`. Split. Exact (Zgt_lt x y).
+ Intros. Apply iff_trans with `y < x`. Split. Exact (Zgt_lt x y).
Exact (Zlt_gt y x).
Exact (Zlt_is_le_bool y x).
Qed.