aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapList.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-09 15:42:09 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-09 15:42:09 +0000
commitf5c21623a1de473b825716c98ab48bfb4776d9a1 (patch)
tree6b906f07fd00cac90e92c9f2677a5c69075c7788 /theories/FSets/FMapList.v
parentdbf346a26275f8c748727d738801efe2d91c7a4f (diff)
Argument Scope de list déplacé dans List.v
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9035 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapList.v')
-rw-r--r--theories/FSets/FMapList.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/theories/FSets/FMapList.v b/theories/FSets/FMapList.v
index 1b40b09f2..86f1dfdc2 100644
--- a/theories/FSets/FMapList.v
+++ b/theories/FSets/FMapList.v
@@ -20,8 +20,6 @@ Require Import FMapInterface.
Set Implicit Arguments.
Unset Strict Implicit.
-Arguments Scope list [type_scope].
-
Module Raw (X:OrderedType).
Module E := X.