src/HOL/Induct/Com.thy
changeset 24178 4ff1dc2aa18d
parent 23746 a455e69c31cc
child 24824 b7866aea0815
--- a/src/HOL/Induct/Com.thy	Tue Aug 07 20:19:54 2007 +0200
+++ b/src/HOL/Induct/Com.thy	Tue Aug 07 20:19:55 2007 +0200
@@ -93,10 +93,7 @@
   "((\<lambda>x x' y. ((x, x'), y) \<in> R) <= (\<lambda>x x' y. ((x, x'), y) \<in> S)) = (R <= S)"
   by (auto simp add: le_fun_def le_bool_def)
 
-ML {*
-Unify.trace_bound := 30;
-Unify.search_bound := 60;
-*}
+declare [[unify_trace_bound = 30, unify_search_bound = 60]]
 
 text{*Command execution is functional (deterministic) provided evaluation is*}
 theorem single_valued_exec: "single_valued ev ==> single_valued(exec ev)"