From eaa3f9719d6190ba92ce55816f11c70b30434309 Mon Sep 17 00:00:00 2001 From: Nickolai Zeldovich Date: Sun, 9 Nov 2014 18:32:55 -0500 Subject: Prove [map_ext] using [map_ext_in]. Since [map_ext_in] is more general, no need to have the same proof twice. --- theories/Lists/List.v | 13 ++++++------- 1 file changed, 6 insertions(+), 7 deletions(-) (limited to 'theories/Lists') diff --git a/theories/Lists/List.v b/theories/Lists/List.v index 00406f57d..ea07a8497 100644 --- a/theories/Lists/List.v +++ b/theories/Lists/List.v @@ -1014,13 +1014,6 @@ Proof. rewrite IHl; auto. Qed. -Lemma map_ext : - forall (A B : Type)(f g:A->B), (forall a, f a = g a) -> forall l, map f l = map g l. -Proof. - induction l; simpl; auto. - rewrite H; rewrite IHl; auto. -Qed. - Lemma map_ext_in : forall (A B : Type)(f g:A->B) l, (forall a, In a l -> f a = g a) -> map f l = map g l. Proof. @@ -1028,6 +1021,12 @@ Proof. intros; rewrite H by intuition; rewrite IHl; auto. Qed. +Lemma map_ext : + forall (A B : Type)(f g:A->B), (forall a, f a = g a) -> forall l, map f l = map g l. +Proof. + intros; apply map_ext_in; auto. +Qed. + (************************************) (** Left-to-right iterator on lists *) -- cgit v1.2.3