src/HOL/ex/CodeEval.thy
changeset 20453 855f07fabd76
parent 20435 d2a30fed7596
child 20597 65fe827aa595
--- a/src/HOL/ex/CodeEval.thy	Thu Aug 31 23:01:16 2006 +0200
+++ b/src/HOL/ex/CodeEval.thy	Fri Sep 01 08:36:51 2006 +0200
@@ -194,7 +194,7 @@
 and ('a, 'b) cair =
     Cair 'a 'b
 
-code_generate term_of
+code_gen term_of
 
 ML {* Eval.term "Shift (Cair (4::nat) [Suc 0])" *}