aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zcompare.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-23 16:35:22 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-23 16:35:22 +0000
commit485151f9ee054b0a0f390d4eff6a2bb2958ed8c2 (patch)
treebf20496ba0e5a17e072517dcbfed18fe9e1b7560 /theories/ZArith/Zcompare.v
parent3d05401764a747c9afbfd950e51e0f0b28a1349c (diff)
Some more cleanup of Zorder
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14234 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zcompare.v')
-rw-r--r--theories/ZArith/Zcompare.v18
1 files changed, 10 insertions, 8 deletions
diff --git a/theories/ZArith/Zcompare.v b/theories/ZArith/Zcompare.v
index 25925a25c..20e1b006a 100644
--- a/theories/ZArith/Zcompare.v
+++ b/theories/ZArith/Zcompare.v
@@ -7,12 +7,15 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(**********************************************************************)
-(** Binary Integers (Pierre Crégut, CNET, Lannion, France) *)
-(**********************************************************************)
+(** Binary Integers : results about Zcompare *)
+(** Initial author: Pierre Crégut (CNET, Lannion, France *)
+
+(** THIS FILE IS DEPRECATED.
+ It is now almost entirely made of compatibility formulations
+ for results already present in BinInt.Z. *)
Require Export BinPos BinInt.
-Require Import Lt Gt Plus Mult. (* Useless now, for compatibility *)
+Require Import Lt Gt Plus Mult. (* Useless now, for compatibility only *)
Local Open Scope Z_scope.
@@ -35,7 +38,7 @@ Lemma Zcompare_Gt_trans :
forall n m p:Z, (n ?= m) = Gt -> (m ?= p) = Gt -> (n ?= p) = Gt.
Proof.
intros n m p. change (n > m -> m > p -> n > p).
- rewrite !Z.gt_lt_iff. intros. now transitivity m.
+ Z.swap_greater. intros. now transitivity m.
Qed.
(** * Comparison and opposite *)
@@ -75,8 +78,7 @@ Qed.
Lemma Zcompare_Gt_not_Lt n m : (n ?= m) = Gt <-> (n ?= m+1) <> Lt.
Proof.
- change (n > m <-> n >= m+1). rewrite Z.gt_lt_iff, Z.ge_le_iff.
- symmetry. apply Z.le_succ_l.
+ change (n > m <-> n >= m+1). Z.swap_greater. symmetry. apply Z.le_succ_l.
Qed.
(** * Successor and comparison *)
@@ -119,7 +121,7 @@ Lemma Zcompare_elim :
| Gt => c3
end.
Proof.
- intros. case Z.compare_spec; trivial. now rewrite <- Z.gt_lt_iff.
+ intros. case Z.compare_spec; trivial. now Z.swap_greater.
Qed.
Lemma Zcompare_eq_case :