From da178a880e3ace820b41d38b191d3785b82991f5 Mon Sep 17 00:00:00 2001 From: Stephane Glondu Date: Thu, 1 Jul 2010 17:21:14 +0200 Subject: Imported Upstream version 8.2pl2+dfsg --- theories/Lists/List.v | 8 ++++---- 1 file changed, 4 insertions(+), 4 deletions(-) (limited to 'theories/Lists/List.v') diff --git a/theories/Lists/List.v b/theories/Lists/List.v index a72283d9..c015854e 100644 --- a/theories/Lists/List.v +++ b/theories/Lists/List.v @@ -6,7 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: List.v 10999 2008-05-27 15:55:22Z letouzey $ i*) +(*i $Id: List.v 12446 2009-10-29 21:43:06Z glondu $ i*) Require Import Le Gt Minus Min Bool. @@ -1081,11 +1081,11 @@ Section Map. (** [flat_map] *) - Fixpoint flat_map (f:A -> list B) (l:list A) {struct l} : - list B := + Definition flat_map (f:A -> list B) := + fix flat_map (l:list A) {struct l} : list B := match l with | nil => nil - | cons x t => (f x)++(flat_map f t) + | cons x t => (f x)++(flat_map t) end. Lemma in_flat_map : forall (f:A->list B)(l:list A)(y:B), -- cgit v1.2.3