src/HOLCF/Lift.thy
changeset 16121 a80aa66d2271
parent 16067 c57725e8055a
child 16216 279ab2e02089
--- a/src/HOLCF/Lift.thy	Tue May 31 11:53:11 2005 +0200
+++ b/src/HOLCF/Lift.thy	Tue May 31 11:53:12 2005 +0200
@@ -165,7 +165,7 @@
   For @{term "x ~= UU"} in assumptions @{text def_tac} replaces @{text
   x} by @{text "Def a"} in conclusion. *}
 
-ML_setup {*
+ML {*
   local val not_Undef_is_Def = thm "not_Undef_is_Def"
   in val def_tac = SIMPSET' (fn ss =>
     etac (not_Undef_is_Def RS iffD1 RS exE) THEN' asm_simp_tac ss)
@@ -268,7 +268,7 @@
   cont_flift1_arg_and_not_arg cont2cont_CF1L_rev2
   cont_Rep_CFun_app cont_Rep_CFun_app_app cont_if
 
-ML_setup {*
+ML {*
 val cont_lemmas2 = cont_lemmas1 @ thms "cont_lemmas_ext";
 
 fun cont_tac  i = resolve_tac cont_lemmas2 i;