summaryrefslogtreecommitdiff
path: root/backend/Kildall.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2007-03-05 08:56:42 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2007-03-05 08:56:42 +0000
commit4d0036dbe756e00627b7185ce8a69984405e062c (patch)
treee8b0fc75221223a70aed1d422c1d44f36b53e967 /backend/Kildall.v
parentc98440cad6b7a9c793aded892ec61a8ed50cac28 (diff)
Importer OrderedPositive depuis Ordered.v
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@183 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'backend/Kildall.v')
-rw-r--r--backend/Kildall.v31
1 files changed, 1 insertions, 30 deletions
diff --git a/backend/Kildall.v b/backend/Kildall.v
index 2a4b4bd..4379b00 100644
--- a/backend/Kildall.v
+++ b/backend/Kildall.v
@@ -1101,36 +1101,7 @@ End BBlock_solver.
Require Import FSets.
Require Import FSetAVL.
-
-Module OrderedPositive <: OrderedType with Definition t := positive.
- Definition t := positive.
- Definition eq (x y: t) := x = y.
- Definition lt := Plt.
-
- Lemma eq_refl : forall x : t, eq x x.
- Proof. unfold eq; auto. Qed.
-
- Lemma eq_sym : forall x y : t, eq x y -> eq y x.
- Proof. unfold eq; auto. Qed.
-
- Lemma eq_trans : forall x y z : t, eq x y -> eq y z -> eq x z.
- Proof. unfold eq; intros. transitivity y; auto. Qed.
-
- Lemma lt_trans : forall x y z : t, lt x y -> lt y z -> lt x z.
- Proof Plt_trans.
-
- Lemma lt_not_eq : forall x y : t, lt x y -> ~ eq x y.
- Proof Plt_ne.
-
- Lemma compare : forall x y : t, Compare lt eq x y.
- Proof.
- intros.
- caseEq (Zcompare (Zpos x) (Zpos y)); intros.
- apply EQ. unfold eq. generalize (Zcompare_Eq_eq _ _ H). congruence.
- apply LT. exact H.
- apply GT. rewrite Zcompare_Gt_Lt_antisym in H. exact H.
- Qed.
-End OrderedPositive.
+Require Import Ordered.
Module PositiveSet := FSetAVL.Make(OrderedPositive).
Module PositiveSetFacts := FSetFacts.Facts(PositiveSet).