src/HOL/Code_Eval.thy
changeset 31998 2c7a24f74db9
parent 31746 75fe3304015c
child 32069 6d28bbd33e2c
--- a/src/HOL/Code_Eval.thy	Tue Jul 14 10:53:44 2009 +0200
+++ b/src/HOL/Code_Eval.thy	Tue Jul 14 10:54:04 2009 +0200
@@ -32,7 +32,7 @@
   \<Rightarrow> 'a \<times> (unit \<Rightarrow> term) \<Rightarrow> 'b \<times> (unit \<Rightarrow> term)" where
   "valapp f x = (fst f (fst x), \<lambda>u. App (snd f ()) (snd x ()))"
 
-lemma valapp_code [code, code inline]:
+lemma valapp_code [code, code_inline]:
   "valapp (f, tf) (x, tx) = (f x, \<lambda>u. App (tf ()) (tx ()))"
   by (simp only: valapp_def fst_conv snd_conv)