aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zmax.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-27 08:31:45 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-27 08:31:45 +0000
commit42331c8a1f29b97b6fa3300a667eea57deac86d0 (patch)
tree994af72db1a54108fcab8f5607352f2a77f4ae34 /theories/ZArith/Zmax.v
parent09db4999b6fd09dd33ccdd423f72b86d1eb9fe86 (diff)
Add a few properties about Rmin/Rmax with replication in Zmin/Zmax.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12358 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zmax.v')
-rw-r--r--theories/ZArith/Zmax.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/theories/ZArith/Zmax.v b/theories/ZArith/Zmax.v
index 413b685a2..b7911181f 100644
--- a/theories/ZArith/Zmax.v
+++ b/theories/ZArith/Zmax.v
@@ -81,6 +81,11 @@ Proof.
intros; apply Zmax_case; assumption.
Qed.
+Lemma Zmax_lub_lt : forall n m p:Z, n < p -> m < p -> Zmax n m < p.
+Proof.
+ intros; apply Zmax_case; assumption.
+Qed.
+
(** * Semi-lattice properties of max *)
Lemma Zmax_idempotent : forall n:Z, Zmax n n = n.