aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/PolyList.v
diff options
context:
space:
mode:
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)).