aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/stdlib
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-08 16:00:09 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-08 16:00:09 +0000
commitf57f892e4dd927acea4cf4bb3816a831e8f90dd2 (patch)
tree5bec19236caa3e912b03d693db9f49695078a4d6 /doc/stdlib
parentd1be0ed0d067dc37afcc5db5e58cee5c2a89d646 (diff)
updates concerning FSets
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10527 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/stdlib')
-rw-r--r--doc/stdlib/index-list.html.template18
1 files changed, 6 insertions, 12 deletions
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template
index ba306b887..aa725b948 100644
--- a/doc/stdlib/index-list.html.template
+++ b/doc/stdlib/index-list.html.template
@@ -309,7 +309,8 @@ through the <tt>Require Import</tt> command.</p>
<dt> <b>IntMap</b>:
- An implementation of finite sets/maps as trees indexed by addresses
+ An implementation of finite sets/maps as trees indexed by
+ addresses (obsolete, supersided by FSets/FMap)
</dt>
<dd>
theories/IntMap/Adalloc.v
@@ -328,7 +329,8 @@ through the <tt>Require Import</tt> command.</p>
</dd>
<dt> <b>FSets</b>:
- Modular implementation of finite sets/maps using lists
+ Modular implementation of finite sets/maps using lists or
+ efficient trees
</dt>
<dd>
theories/FSets/OrderedType.v
@@ -336,18 +338,14 @@ through the <tt>Require Import</tt> command.</p>
theories/FSets/OrderedTypeEx.v
theories/FSets/FSetInterface.v
theories/FSets/FSetBridge.v
+ theories/FSets/FSetFacts.v
theories/FSets/FSetProperties.v
theories/FSets/FSetEqProperties.v
theories/FSets/FSetList.v
+ theories/FSets/FSetWeakList.v
(theories/FSets/FSets.v)
- theories/FSets/FSetFacts.v
theories/FSets/FSetAVL.v
theories/FSets/FSetToFiniteSet.v
- theories/FSets/FSetWeakProperties.v
- theories/FSets/FSetWeakInterface.v
- theories/FSets/FSetWeakFacts.v
- theories/FSets/FSetWeakList.v
- theories/FSets/FSetWeak.v
theories/FSets/FMapInterface.v
theories/FSets/FMapList.v
theories/FSets/FMapPositive.v
@@ -355,10 +353,6 @@ through the <tt>Require Import</tt> command.</p>
theories/FSets/FMapFacts.v
(theories/FSets/FMaps.v)
theories/FSets/FMapAVL.v
- theories/FSets/FMapWeakInterface.v
- theories/FSets/FMapWeakList.v
- theories/FSets/FMapWeak.v
- theories/FSets/FMapWeakFacts.v
</dd>
<!-- <dt> <b>Strings</b>