aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/PolyList.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-13 16:26:26 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-08-13 16:26:26 +0000
commit8c67206c70ed7fdfd4dc9847e2fb11cff77df968 (patch)
tree1bc5b27e49b2244af1c5ee663fa05056c452a113 /theories/Lists/PolyList.v
parent7a63d8f5df7ae27038c6c770c22ee3911781de85 (diff)
Rétablissement nom de section Map après résolution bugs surcharge de noms
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1898 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/PolyList.v')
-rw-r--r--theories/Lists/PolyList.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Lists/PolyList.v b/theories/Lists/PolyList.v
index 7eeeb73f0..3e845fb88 100644
--- a/theories/Lists/PolyList.v
+++ b/theories/Lists/PolyList.v
@@ -549,7 +549,7 @@ Section Functions_on_lists.
(* Some generic functions on lists and basic functions of them *)
(***************************************************************)
-Section Map_def.
+Section Map.
Variables A,B:Set.
Variable f:A->B.
Fixpoint map [l:(list A)] : (list B) :=
@@ -557,7 +557,7 @@ Fixpoint map [l:(list A)] : (list B) :=
nil => (nil B)
| (cons a t) => (cons (f a) (map t))
end.
-End Map_def.
+End Map.
Lemma in_map : (A,B:Set)(f:A->B)(l:(list A))(x:A)
(In x l) -> (In (f x) (map f l)).