aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zorder.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-12-12 10:38:20 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-12-12 10:38:20 +0000
commitd2d0b966db4b899ac46d57e6f39b5c3b8c5c3753 (patch)
tree5d49b3954d68da5b00b51454840c80a4eaaf546e /theories/ZArith/Zorder.v
parente9d9c0e5394de0fc831f392bb64908a5724e688d (diff)
Bug nommage Zgt_trans_succ
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9438 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zorder.v')
-rw-r--r--theories/ZArith/Zorder.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zorder.v b/theories/ZArith/Zorder.v
index 4b0d2562e..45369561d 100644
--- a/theories/ZArith/Zorder.v
+++ b/theories/ZArith/Zorder.v
@@ -549,7 +549,7 @@ Hint Immediate Zeq_le: zarith.
(** Transitivity using successor *)
-Lemma Zge_trans_succ : forall n m p:Z, Zsucc n > m -> m > p -> n > p.
+Lemma Zgt_trans_succ : forall n m p:Z, Zsucc n > m -> m > p -> n > p.
Proof.
intros n m p H1 H2; apply Zle_gt_trans with (m := m);
[ apply Zgt_succ_le; assumption | assumption ].