src/HOL/Product_Type.thy
changeset 41505 6d19301074cf
parent 41372 551eb49a6e91
child 41792 ff3cb0c418b7
--- a/src/HOL/Product_Type.thy	Mon Jan 10 22:03:24 2011 +0100
+++ b/src/HOL/Product_Type.thy	Tue Jan 11 14:12:37 2011 +0100
@@ -834,7 +834,7 @@
   "map_pair f g (a, b) = (f a, g b)"
   by (simp add: map_pair_def)
 
-type_lifting map_pair: map_pair
+enriched_type map_pair: map_pair
   by (auto simp add: split_paired_all intro: ext)
 
 lemma fst_map_pair [simp]: