aboutsummaryrefslogtreecommitdiffstats
path: root/lib/HashedSet.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-03-05 16:57:54 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-03-05 16:57:54 +0100
commit78c4974c0a362cd0ab3bbd80203c0277d267afbb (patch)
tree225700cd45255386d154044976827c0af0ecc408 /lib/HashedSet.v
parent660c1ec3bb6e52720660d6fbb054884b12dca9ca (diff)
downloadcompcert-kvx-78c4974c0a362cd0ab3bbd80203c0277d267afbb.tar.gz
compcert-kvx-78c4974c0a362cd0ab3bbd80203c0277d267afbb.zip
streamlined lattice code
Diffstat (limited to 'lib/HashedSet.v')
-rw-r--r--lib/HashedSet.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/lib/HashedSet.v b/lib/HashedSet.v
index 6130ba17..2a798727 100644
--- a/lib/HashedSet.v
+++ b/lib/HashedSet.v
@@ -3,6 +3,8 @@ Require Import Bool.
Require Import List.
Require Coq.Logic.Eqdep_dec.
+Require Extraction.
+
Module Type POSITIVE_SET.
Parameter t : Type.
Parameter empty : t.
@@ -116,7 +118,7 @@ Axiom gfilter:
End POSITIVE_SET.
-Module PSet <: POSITIVE_SET.
+Module PSet : POSITIVE_SET.
(* begin from Maps *)
Fixpoint prev_append (i j: positive) {struct i} : positive :=
match i with
@@ -1382,10 +1384,8 @@ Proof.
intros.
apply WR.gfilter.
Qed.
-End PSet.
-Require Extraction.
-
-Extract Inductive PSet.WR.pset => "HashedSetaux.pset" [ "HashedSetaux.empty" "HashedSetaux.node" ] "HashedSetaux.pset_match".
+Extract Inductive WR.pset => "HashedSetaux.pset" [ "HashedSetaux.empty" "HashedSetaux.node" ] "HashedSetaux.pset_match".
-Extract Inlined Constant PSet.WR.pset_eq => "HashedSetaux.eq".
+Extract Inlined Constant WR.pset_eq => "HashedSetaux.eq".
+End PSet.