aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Le.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-27 09:02:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-27 09:02:29 +0000
commitc06d6bd8949a34c1232d2011a3614fa53db84b7d (patch)
tree6095a5ddf865b9456a19a31542bae1f87b90d14b /theories/Arith/Le.v
parentf89026ecf32f696d2036dd1b33766b050ad236c9 (diff)
Bug du commit precedent
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4716 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Le.v')
-rwxr-xr-xtheories/Arith/Le.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Le.v b/theories/Arith/Le.v
index c0a81d23e..71b020e6a 100755
--- a/theories/Arith/Le.v
+++ b/theories/Arith/Le.v
@@ -20,7 +20,7 @@ Theorem le_trans : (n,m,p:nat)(le n m)->(le m p)->(le n p).
Proof.
NewInduction 2; Auto.
Qed.
-Hints Immediate le_trans : arith v62.
+Hints Resolve le_trans : arith v62.
(** Order, successor and predecessor *)