diff -r 46c0c741c8c2 -r 98370b26c2ce src/HOL/Typerep.thy --- a/src/HOL/Typerep.thy Tue May 19 13:57:51 2009 +0200 +++ b/src/HOL/Typerep.thy Tue May 19 16:54:55 2009 +0200 @@ -6,7 +6,7 @@ imports Plain String begin -datatype typerep = Typerep message_string "typerep list" +datatype typerep = Typerep String.literal "typerep list" class typerep = fixes typerep :: "'a itself \ typerep" @@ -45,7 +45,7 @@ val ty = Type (tyco, map TFree vs); val lhs = Const (@{const_name typerep}, Term.itselfT ty --> @{typ typerep}) $ Free ("T", Term.itselfT ty); - val rhs = @{term Typerep} $ HOLogic.mk_message_string tyco + val rhs = @{term Typerep} $ HOLogic.mk_literal tyco $ HOLogic.mk_list @{typ typerep} (map (HOLogic.mk_typerep o TFree) vs); val eq = HOLogic.mk_Trueprop (HOLogic.mk_eq (lhs, rhs)); in