src/HOL/Library/Eval.thy
changeset 24994 c385c4eabb3b
parent 24920 2a45e400fdad
child 25502 9200b36280c0
--- a/src/HOL/Library/Eval.thy	Fri Oct 12 08:20:46 2007 +0200
+++ b/src/HOL/Library/Eval.thy	Fri Oct 12 08:21:09 2007 +0200
@@ -146,9 +146,9 @@
   "term_of k \<equiv> STR ''Numeral.number_class.number_of'' \<Colon>\<subseteq> intT \<rightarrow> intT \<bullet> mk_int k" ..
 
 
-text {* Adaption for @{typ ml_string}s *}
+text {* Adaption for @{typ message_string}s *}
 
-lemmas [code func, code func del] = term_of_ml_string_def
+lemmas [code func, code func del] = term_of_message_string_def
 
 
 subsection {* Evaluation infrastructure *}