src/HOL/ATP_Linkup.thy
changeset 24742 73b8b42a36b6
parent 24318 2477286fcc7e
child 24819 7d8e0a47392e
--- a/src/HOL/ATP_Linkup.thy	Thu Sep 27 17:28:05 2007 +0200
+++ b/src/HOL/ATP_Linkup.thy	Thu Sep 27 17:55:28 2007 +0200
@@ -7,7 +7,8 @@
 header{* The Isabelle-ATP Linkup *}
 
 theory ATP_Linkup
-imports Divides Record Hilbert_Choice
+imports Divides Record Hilbert_Choice Presburger Relation_Power SAT Recdef Extraction 
+   (*It must be a parent or a child of every other theory, to prevent theory-merge errors.*)
 uses
   "Tools/polyhash.ML"
   "Tools/res_clause.ML"
@@ -110,4 +111,11 @@
 use "Tools/metis_tools.ML"
 setup MetisTools.setup
 
+(*Sledgehammer*)
+setup ResAxioms.setup
+
+setup {*
+  Theory.at_end ResAxioms.clause_cache_endtheory
+*}
+
 end