aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-17 17:06:21 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-18 10:26:21 +0100
commit30a9a27ce3a76e2704671174483d4b4f84c482e4 (patch)
treec4788d01c2ff18154877439a793b519f943d5233 /theories/Lists
parent52f51fb385d6a1c90bd7d055185fee50ef2670be (diff)
Clarifying the role of ListSet.v in the library, compared to other
finite set libraries.
Diffstat (limited to 'theories/Lists')
-rw-r--r--theories/Lists/ListSet.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index f02c1d13f..908731117 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -6,11 +6,13 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(** A Library for finite sets, implemented as lists *)
+(** A library for finite sets, implemented as lists *)
-(** List is loaded, but not exported.
- This allow to "hide" the definitions, functions and theorems of List
- and to see only the ones of ListSet *)
+(** This is a light implementation of finite sets as lists; for a more
+ extensive library, you might rather consider MSetWeakList.v. In
+ addition, if your domain is totally ordered, you might also
+ consider implementations of finite sets with access in logarithmic
+ time (e.g. MSetRBT.v which is based on red-black trees). *)
Require Import List.