no setup is necessary anymore
authorblanchet
Mon, 28 Jun 2010 18:47:07 +0200
changeset 37622 b3f572839570
parent 37621 3e78dbf7a382
child 37623 295f3a9b44b6
no setup is necessary anymore
src/HOL/Metis_Examples/Tarski.thy
src/HOL/Sledgehammer.thy
--- a/src/HOL/Metis_Examples/Tarski.thy	Mon Jun 28 18:46:42 2010 +0200
+++ b/src/HOL/Metis_Examples/Tarski.thy	Mon Jun 28 18:47:07 2010 +0200
@@ -507,9 +507,8 @@
 
 (*never proved, 2007-01-22*)
 declare [[ atp_problem_prefix = "Tarski__CLF_lubH_is_fixp" ]]
-(*Single-step version fails. The conjecture clauses refer to local abstraction
-functions (Frees), which prevents expand_defs_tac from removing those 
-"definitions" at the end of the proof. *)
+(* Single-step version fails. The conjecture clauses refer to local abstraction
+functions (Frees). *)
 lemma (in CLF) lubH_is_fixp:
      "H = {x. (x, f x) \<in> r & x \<in> A} ==> lub H cl \<in> fix f A"
 apply (simp add: fix_def)
--- a/src/HOL/Sledgehammer.thy	Mon Jun 28 18:46:42 2010 +0200
+++ b/src/HOL/Sledgehammer.thy	Mon Jun 28 18:47:07 2010 +0200
@@ -86,8 +86,6 @@
 done
 
 use "Tools/Sledgehammer/clausifier.ML"
-setup Clausifier.setup
-
 use "Tools/Sledgehammer/meson_tactic.ML"
 setup Meson_Tactic.setup