aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapInterface.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-21 00:03:14 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-21 00:03:14 +0000
commit7109daa08ff5be5bf28902d9b060cccf73375b4e (patch)
tree7c85db35aaea76d402232d5545a1742a9088dbeb /theories/FSets/FMapInterface.v
parent97b74d43fe5f6070992c4824f823a9725620944e (diff)
Cleanup attempt of Hints in *Interface.v files.
See recent discussion in coq-club. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10243 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapInterface.v')
-rw-r--r--theories/FSets/FMapInterface.v19
1 files changed, 9 insertions, 10 deletions
diff --git a/theories/FSets/FMapInterface.v b/theories/FSets/FMapInterface.v
index 0bd2c4525..d4e07461c 100644
--- a/theories/FSets/FMapInterface.v
+++ b/theories/FSets/FMapInterface.v
@@ -12,12 +12,9 @@
(** This file proposes an interface for finite maps *)
-(* begin hide *)
-Require Export Bool.
-Require Export OrderedType.
+Require Export Bool OrderedType.
Set Implicit Arguments.
Unset Strict Implicit.
-(* end hide *)
(** When compared with Ocaml Map, this signature has been split in two:
- The first part [S] contains the usual operators (add, find, ...)
@@ -206,12 +203,14 @@ Module Type S.
(x:key)(f:option elt->option elt'->option elt''),
In x (map2 f m m') -> In x m \/ In x m'.
- (* begin hide *)
- Hint Immediate MapsTo_1 mem_2 is_empty_2.
-
- Hint Resolve mem_1 is_empty_1 is_empty_2 add_1 add_2 add_3 remove_1
- remove_2 remove_3 find_1 find_2 fold_1 map_1 map_2 mapi_1 mapi_2.
- (* end hide *)
+ Hint Immediate MapsTo_1 mem_2 is_empty_2
+ map_2 mapi_2 add_3 remove_3 find_2
+ : map.
+ Hint Resolve mem_1 is_empty_1 is_empty_2 add_1 add_2 remove_1
+ remove_2 find_1 fold_1 map_1 mapi_1 mapi_2
+ : map.
+ (** for compatibility with earlier hints *)
+ Hint Resolve map_2 mapi_2 add_3 remove_3 find_2 : oldmap.
End S.