diff -r a7462e442e35 -r 6d19301074cf src/HOL/List.thy --- a/src/HOL/List.thy Mon Jan 10 22:03:24 2011 +0100 +++ b/src/HOL/List.thy Tue Jan 11 14:12:37 2011 +0100 @@ -880,7 +880,7 @@ "length xs = length ys \ map snd (zip xs ys) = ys" by (induct rule:list_induct2, simp_all) -type_lifting map: map +enriched_type map: map by (simp_all add: fun_eq_iff id_def)