src/HOL/Product_Type.thy
changeset 40968 a6fcd305f7dc
parent 40929 7ff03a5e044f
child 41229 d797baa3d57c
--- a/src/HOL/Product_Type.thy	Sun Dec 05 14:02:16 2010 +0100
+++ b/src/HOL/Product_Type.thy	Mon Dec 06 09:19:10 2010 +0100
@@ -835,7 +835,7 @@
   "map_pair f g (a, b) = (f a, g b)"
   by (simp add: map_pair_def)
 
-type_mapper map_pair
+type_lifting map_pair
   by (simp_all add: split_paired_all)
 
 lemma fst_map_pair [simp]: