aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapWeakList.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-05 16:31:16 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-05 16:31:16 +0000
commit316e114dd188f85ec657420989bf909ecfe9d006 (patch)
tree37229712b18593049740b28b6a18a5d9e7150faa /theories/FSets/FMapWeakList.v
parent44cedab7be5a44a01d467fbd2dba24400d575206 (diff)
kill some useless module aliases E:=X (for better name printing, see Elie's 14097)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10511 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapWeakList.v')
-rw-r--r--theories/FSets/FMapWeakList.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/FSets/FMapWeakList.v b/theories/FSets/FMapWeakList.v
index 579fd50c9..0dcfb05f3 100644
--- a/theories/FSets/FMapWeakList.v
+++ b/theories/FSets/FMapWeakList.v
@@ -11,7 +11,7 @@
(** * Finite map library *)
(** This file proposes an implementation of the non-dependant interface
- [FMapInterface.WS] using lists of pairs, unordered but without redundancy. *)
+ [FMapInterface.WS] using lists of pairs, unordered but without redundancy. *)
Require Import FMapInterface.