src/HOL/Record.thy
changeset 58152 6fe60a9a5bad
parent 56732 da3fefcb43c3
child 58310 91ea607a34d8
--- a/src/HOL/Record.thy	Wed Sep 03 00:06:23 2014 +0200
+++ b/src/HOL/Record.thy	Wed Sep 03 00:06:24 2014 +0200
@@ -79,7 +79,7 @@
 
 subsection {* Operators and lemmas for types isomorphic to tuples *}
 
-datatype ('a, 'b, 'c) tuple_isomorphism =
+datatype_new (dead 'a, dead 'b, dead 'c) tuple_isomorphism =
   Tuple_Isomorphism "'a \<Rightarrow> 'b \<times> 'c" "'b \<times> 'c \<Rightarrow> 'a"
 
 primrec