aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-20 17:18:44 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-20 17:18:44 +0000
commitc251e659c18859d0d8522781ff9d95723b253c11 (patch)
tree8ef519455696d0ef4f5535daa1c347261960d64f /theories/ZArith
parent946adf37ceb99d84e7b96211bfdbd0ba2d134a01 (diff)
Zcompare.destr_zcompare subsumed by case Z.compare_spec
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14229 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith')
-rw-r--r--theories/ZArith/Zcompare.v9
1 files changed, 0 insertions, 9 deletions
diff --git a/theories/ZArith/Zcompare.v b/theories/ZArith/Zcompare.v
index 49ab619bc..25925a25c 100644
--- a/theories/ZArith/Zcompare.v
+++ b/theories/ZArith/Zcompare.v
@@ -19,15 +19,6 @@ Local Open Scope Z_scope.
(***************************)
(** * Comparison on integers *)
-Ltac destr_zcompare :=
- match goal with |- context [Z.compare ?x ?y] =>
- let H := fresh "H" in
- case_eq (Z.compare x y); intro H;
- [generalize (Z.compare_eq _ _ H); clear H; intro H |
- change (x<y)%Z in H |
- change (x>y)%Z in H ]
- end.
-
Lemma Zcompare_Gt_Lt_antisym : forall n m:Z, (n ?= m) = Gt <-> (m ?= n) = Lt.
Proof Z.gt_lt_iff.