aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/BinInt.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/BinInt.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/BinInt.v')
-rw-r--r--theories/ZArith/BinInt.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/theories/ZArith/BinInt.v b/theories/ZArith/BinInt.v
index d07fe5174..673276d3e 100644
--- a/theories/ZArith/BinInt.v
+++ b/theories/ZArith/BinInt.v
@@ -1261,6 +1261,10 @@ Proof.
apply ge_le_iff.
Qed.
+(** We provide a tactic converting from one style to the other. *)
+
+Ltac swap_greater := rewrite ?gt_lt_iff in *; rewrite ?ge_le_iff in *.
+
(** Similarly, the boolean comparisons [ltb] and [leb] are favored
over their dual [gtb] and [geb]. We prove here the equivalence
and a few minimal results. *)