diff -r cace30ea5a2c -r 85f944352d55 src/HOL/Metis_Examples/Clausification.thy --- a/src/HOL/Metis_Examples/Clausification.thy Thu Jan 03 13:11:04 2013 +0100 +++ b/src/HOL/Metis_Examples/Clausification.thy Thu Jan 03 13:28:37 2013 +0100 @@ -10,10 +10,6 @@ imports Complex_Main begin -(* FIXME: shouldn't need this *) -declare [[unify_search_bound = 100]] -declare [[unify_trace_bound = 100]] - text {* Definitional CNF for facts *} @@ -139,7 +135,7 @@ lemma "(\x \ set xs. P x) \ (\ys x zs. xs = ys @ x # zs \ P x \ (\z \ set zs. \ P z))" -by (metis split_list_last_prop [where P = P] in_set_conv_decomp) +by (metis split_list_last_prop[where P = P] in_set_conv_decomp) lemma ex_tl: "EX ys. tl ys = xs" using tl.simps(2) by fast