From 8c67206c70ed7fdfd4dc9847e2fb11cff77df968 Mon Sep 17 00:00:00 2001 From: herbelin Date: Mon, 13 Aug 2001 16:26:26 +0000 Subject: Rétablissement nom de section Map après résolution bugs surcharge de noms MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1898 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Lists/PolyList.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/Lists/PolyList.v') 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)). -- cgit v1.2.3