aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith/Qround.v
diff options
context:
space:
mode:
authorGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-05 10:47:51 +0000
committerGravatar roconnor <roconnor@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-05 10:47:51 +0000
commit362ccc063fa14ee0dbec6f25f1d4c45eca11013a (patch)
treeae298ffa18564d4cf3ff0fd48da6605b72b6a6a5 /theories/QArith/Qround.v
parent2fb65d97bfd9ccba49b6081810f1a72841bb3d55 (diff)
Add Morphisms for Qceiling and Qfloor
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10508 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/QArith/Qround.v')
-rw-r--r--theories/QArith/Qround.v16
1 files changed, 16 insertions, 0 deletions
diff --git a/theories/QArith/Qround.v b/theories/QArith/Qround.v
index 2479c2259..8162a702f 100644
--- a/theories/QArith/Qround.v
+++ b/theories/QArith/Qround.v
@@ -121,3 +121,19 @@ cut (Qfloor (-y) <= Qfloor (-x))%Z; auto with *.
Qed.
Hint Resolve Qceiling_resp_le : qarith.
+
+Add Morphism Qfloor with signature Qeq ==> eq as Qfloor_comp.
+Proof.
+intros x y H.
+apply Zle_antisym.
+ auto with *.
+symmetry in H; auto with *.
+Qed.
+
+Add Morphism Qceiling with signature Qeq ==> eq as Qceiling_comp.
+Proof.
+intros x y H.
+apply Zle_antisym.
+ auto with *.
+symmetry in H; auto with *.
+Qed. \ No newline at end of file