src/HOL/Induct/Com.thy
changeset 32367 a508148f7c25
parent 26806 40b411ec05aa
child 36862 952b2b102a0a
--- a/src/HOL/Induct/Com.thy	Thu Aug 13 17:19:10 2009 +0100
+++ b/src/HOL/Induct/Com.thy	Thu Aug 13 17:19:42 2009 +0100
@@ -91,8 +91,6 @@
   "((\<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 mem_def)
 
-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)"
 apply (simp add: single_valued_def)