From 3a304ad8434e1c4f5428159aaa029f4b7734685e Mon Sep 17 00:00:00 2001 From: letouzey Date: Wed, 19 Mar 2008 21:17:28 +0000 Subject: some references to IntMap forgotten in last commit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10700 85f007b7-540e-0410-9357-904b9bb8a0f7 --- doc/stdlib/index-list.html.template | 22 ---------------------- toplevel/coqinit.ml | 1 - 2 files changed, 23 deletions(-) diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template index aa725b948..c86338175 100644 --- a/doc/stdlib/index-list.html.template +++ b/doc/stdlib/index-list.html.template @@ -307,27 +307,6 @@ through the Require Import command.

theories/Wellfounded/Well_Ordering.v - -
IntMap: - An implementation of finite sets/maps as trees indexed by - addresses (obsolete, supersided by FSets/FMap) -
-
- theories/IntMap/Adalloc.v - theories/IntMap/Map.v - theories/IntMap/Fset.v - theories/IntMap/Mapaxioms.v - theories/IntMap/Mapiter.v - theories/IntMap/Mapcanon.v - theories/IntMap/Mapsubset.v - theories/IntMap/Lsort.v - theories/IntMap/Mapfold.v - theories/IntMap/Mapcard.v - theories/IntMap/Mapc.v - theories/IntMap/Maplists.v - theories/IntMap/Allmaps.v -
-
FSets: Modular implementation of finite sets/maps using lists or efficient trees @@ -349,7 +328,6 @@ through the Require Import command.

theories/FSets/FMapInterface.v theories/FSets/FMapList.v theories/FSets/FMapPositive.v - theories/FSets/FMapIntMap.v theories/FSets/FMapFacts.v (theories/FSets/FMaps.v) theories/FSets/FMapAVL.v diff --git a/toplevel/coqinit.ml b/toplevel/coqinit.ml index 95ffeb44a..10d64dcf8 100644 --- a/toplevel/coqinit.ml +++ b/toplevel/coqinit.ml @@ -74,7 +74,6 @@ let theories_dirs_map = [ "theories/Classes", "Classes" ; "theories/Program", "Program" ; "theories/FSets", "FSets" ; - "theories/IntMap", "IntMap" ; "theories/Reals", "Reals" ; "theories/Strings", "Strings" ; "theories/Sorting", "Sorting" ; -- cgit v1.2.3