src/HOL/Code_Setup.thy
changeset 24835 8c26128f8997
parent 24463 841c2e24761f
child 24844 98c006a30218
--- a/src/HOL/Code_Setup.thy	Thu Oct 04 16:59:30 2007 +0200
+++ b/src/HOL/Code_Setup.thy	Thu Oct 04 19:41:49 2007 +0200
@@ -136,7 +136,7 @@
 subsection {* Evaluation oracle *}
 
 oracle eval_oracle ("term") = {* fn thy => fn t => 
-  if CodePackage.satisfies thy (Thm.cterm_of thy (HOLogic.dest_Trueprop t)) [] 
+  if CodePackage.satisfies thy (HOLogic.dest_Trueprop t) [] 
   then t
   else HOLogic.Trueprop $ HOLogic.true_const (*dummy*)
 *}
@@ -156,7 +156,7 @@
 
 method_setup normalization = {*
   Method.no_args (Method.SIMPLE_METHOD'
-    (CONVERSION (ObjectLogic.judgment_conv Nbe.normalization_conv)
+    (CONVERSION (ObjectLogic.judgment_conv Nbe.norm_conv)
       THEN' resolve_tac [TrueI, refl]))
 *} "solve goal by normalization"