aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapInterface.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-14 21:26:47 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-14 21:26:47 +0000
commit0a74b74e0010e97fbb79d68d0f36ea30cf118aec (patch)
tree548744c12a6d3e8ad0fa99fa5d3ff762930efdf9 /theories/FSets/FMapInterface.v
parent54286eace13cf1f0509e85ff6f47705e741c2b64 (diff)
Rework of FSetProperties, in order to add more easily a Properties functor
for FMap (for the moment in FMapFacts). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9890 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapInterface.v')
-rw-r--r--theories/FSets/FMapInterface.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/FSets/FMapInterface.v b/theories/FSets/FMapInterface.v
index 03c64b1ef..0bd2c4525 100644
--- a/theories/FSets/FMapInterface.v
+++ b/theories/FSets/FMapInterface.v
@@ -13,9 +13,10 @@
(** This file proposes an interface for finite maps *)
(* begin hide *)
+Require Export Bool.
+Require Export OrderedType.
Set Implicit Arguments.
Unset Strict Implicit.
-Require Import FSetInterface.
(* end hide *)
(** When compared with Ocaml Map, this signature has been split in two: