aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Znat.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-03-28 19:35:03 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-03-28 19:35:03 +0000
commit1c4a4908a82e2eba9cc2d335697d51182f7314c2 (patch)
tree39f6a5b7caf7d583af468d59c9f62378a748f8d3 /theories/ZArith/Znat.v
parentbe76b6af359ea61bc71e59efb4802ff01cce728c (diff)
Fixing bug #2254 (inappropriate names of Zlt_gt_succ and Zlt_succ_gt)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12888 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Znat.v')
-rw-r--r--theories/ZArith/Znat.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Znat.v b/theories/ZArith/Znat.v
index 0fc27e38b..dfd9b5450 100644
--- a/theories/ZArith/Znat.v
+++ b/theories/ZArith/Znat.v
@@ -91,7 +91,7 @@ Qed.
Theorem inj_lt : forall n m:nat, (n < m)%nat -> Z_of_nat n < Z_of_nat m.
Proof.
- intros x y H; apply Zgt_lt; apply Zlt_succ_gt; rewrite <- inj_S; apply inj_le;
+ intros x y H; apply Zgt_lt; apply Zle_succ_gt; rewrite <- inj_S; apply inj_le;
exact H.
Qed.