aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/PArith/BinPos.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-11-02 19:30:57 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-11-02 19:30:57 +0000
commit2a7a989025a5dde9a6f34792e1e1f2b4e3ad3108 (patch)
tree63b6bf19f0cf27bfc4a2d77381eef5a0cb403c85 /theories/PArith/BinPos.v
parentc5eea71cebc0fd1553196598e6b88af482dbffe5 (diff)
Add small utility lemmas about nat/P/Z/Q arithmetic.
Initial patch by Eelis van der Weegen, minor adaptations by myself git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13613 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/PArith/BinPos.v')
-rw-r--r--theories/PArith/BinPos.v6
1 files changed, 5 insertions, 1 deletions
diff --git a/theories/PArith/BinPos.v b/theories/PArith/BinPos.v
index 663233c57..9c8775f82 100644
--- a/theories/PArith/BinPos.v
+++ b/theories/PArith/BinPos.v
@@ -1025,6 +1025,11 @@ Proof.
destruct ((p ?= q) Eq); intuition; discriminate.
Qed.
+Lemma Ple_refl : forall p, Ple p p.
+Proof.
+ intros. unfold Ple. rewrite Pcompare_refl_id. discriminate.
+Qed.
+
(** Strict order and operations *)
Lemma Pplus_lt_mono_l : forall p q r, q<r <-> p+q < p+r.
@@ -1070,7 +1075,6 @@ Proof.
apply Plt_trans with (p+q); auto using Plt_plus_r.
Qed.
-
(**********************************************************************)
(** Properties of subtraction on binary positive numbers *)