aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zorder.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/ZArith/Zorder.v')
-rw-r--r--theories/ZArith/Zorder.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/theories/ZArith/Zorder.v b/theories/ZArith/Zorder.v
index 32faf5a95..a8cd69bb3 100644
--- a/theories/ZArith/Zorder.v
+++ b/theories/ZArith/Zorder.v
@@ -111,6 +111,12 @@ Proof.
Z.swap_greater. apply Z.nle_gt.
Qed.
+Lemma not_Zne n m : ~ Zne n m -> n = m.
+Proof.
+ intros H.
+ destruct (Z.eq_decidable n m); [assumption|now elim H].
+Qed.
+
(** * Equivalence and order properties *)
(** Reflexivity *)