From 78c4974c0a362cd0ab3bbd80203c0277d267afbb Mon Sep 17 00:00:00 2001 From: David Monniaux Date: Thu, 5 Mar 2020 16:57:54 +0100 Subject: streamlined lattice code --- lib/HashedSet.v | 12 ++++++------ 1 file changed, 6 insertions(+), 6 deletions(-) (limited to 'lib/HashedSet.v') 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. -- cgit