From f57f892e4dd927acea4cf4bb3816a831e8f90dd2 Mon Sep 17 00:00:00 2001 From: letouzey Date: Fri, 8 Feb 2008 16:00:09 +0000 Subject: updates concerning FSets git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10527 85f007b7-540e-0410-9357-904b9bb8a0f7 --- doc/stdlib/index-list.html.template | 18 ++++++------------ 1 file changed, 6 insertions(+), 12 deletions(-) (limited to 'doc') 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 Require Import command.

IntMap: - 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)
theories/IntMap/Adalloc.v @@ -328,7 +329,8 @@ through the Require Import command.

FSets: - Modular implementation of finite sets/maps using lists + Modular implementation of finite sets/maps using lists or + efficient trees
theories/FSets/OrderedType.v @@ -336,18 +338,14 @@ through the Require Import command.

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 Require Import command.

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