src/HOL/Bali/Term.thy
changeset 24019 67bde7cfcf10
parent 16417 9bc16273c2d4
child 24783 5a3e336a2e37
--- a/src/HOL/Bali/Term.thy	Sat Jul 28 20:40:20 2007 +0200
+++ b/src/HOL/Bali/Term.thy	Sat Jul 28 20:40:22 2007 +0200
@@ -266,9 +266,7 @@
   is_stmt :: "term \<Rightarrow> bool"
  "is_stmt t \<equiv> \<exists>c. t=In1r c"
 
-ML {*
-bind_thms ("is_stmt_rews", sum3_instantiate (thm "is_stmt_def"));
-*}
+ML_setup {* bind_thms ("is_stmt_rews", sum3_instantiate @{thm is_stmt_def}) *}
 
 declare is_stmt_rews [simp]