| changeset 28054 | 2b84d34c5d02 | 
| parent 27487 | c8a6ce181805 | 
| child 28064 | d4a6460c53d1 | 
--- a/src/HOL/Library/Code_Message.thy Thu Aug 28 22:08:11 2008 +0200 +++ b/src/HOL/Library/Code_Message.thy Thu Aug 28 22:09:20 2008 +0200 @@ -51,7 +51,7 @@ @{const_name NibbleC}, @{const_name NibbleD}, @{const_name NibbleE}, @{const_name NibbleF}]; in - fold (fn target => CodeTarget.add_pretty_message target + fold (fn target => Code_Target.add_pretty_message target charr nibbles @{const_name Nil} @{const_name Cons} @{const_name STR}) ["SML", "OCaml", "Haskell"] end