src/HOL/List.thy
changeset 55467 a5c9002bc54d
parent 55466 786edc984c98
child 55473 c582a7893dcd
--- a/src/HOL/List.thy	Fri Feb 14 07:53:46 2014 +0100
+++ b/src/HOL/List.thy	Fri Feb 14 07:53:46 2014 +0100
@@ -1160,7 +1160,7 @@
   "length xs = length ys \<Longrightarrow> map snd (zip xs ys) = ys"
 by (induct rule:list_induct2, simp_all)
 
-enriched_type map: map
+functor map: map
 by (simp_all add: id_def)
 
 declare map.id [simp]