| changeset 28064 | d4a6460c53d1 | 
| parent 28054 | 2b84d34c5d02 | 
| child 28090 | 29af3c712d2b | 
--- a/src/HOL/Library/Code_Message.thy Fri Aug 29 20:36:08 2008 +0200 +++ b/src/HOL/Library/Code_Message.thy Mon Sep 01 10:18:37 2008 +0200 @@ -51,7 +51,7 @@ @{const_name NibbleC}, @{const_name NibbleD}, @{const_name NibbleE}, @{const_name NibbleF}]; in - fold (fn target => Code_Target.add_pretty_message target + fold (fn target => Code_Target.add_literal_message target charr nibbles @{const_name Nil} @{const_name Cons} @{const_name STR}) ["SML", "OCaml", "Haskell"] end