aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetAVL.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-19 20:56:43 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-03-19 20:56:43 +0000
commit509cd11ac957c0ff97cbe9a0cd50852c74095e36 (patch)
treeaeadbbc55f35b9c572a4f76084bb5ec7a5c9e401 /theories/FSets/FSetAVL.v
parent0157aadd967fcba870fb9bf74ea2af7671105efc (diff)
migration of the old IntMap library from StdLib to a user contrib (Cachan/IntMap)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10699 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FSetAVL.v')
-rw-r--r--theories/FSets/FSetAVL.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/FSets/FSetAVL.v b/theories/FSets/FSetAVL.v
index 5973b21ec..024c2e963 100644
--- a/theories/FSets/FSetAVL.v
+++ b/theories/FSets/FSetAVL.v
@@ -37,7 +37,7 @@
code after extraction.
*)
-Require Import Recdef FSetInterface FSetList ZArith Int.
+Require Import FSetInterface FSetList ZArith Int.
Set Implicit Arguments.
Unset Strict Implicit.