src/FOL/IFOL.thy
changeset 30240 5b25fee0362c
parent 28856 5e009a80fe6d
child 30242 aea5d7fa7ef5
--- a/src/FOL/IFOL.thy	Wed Mar 04 10:43:39 2009 +0100
+++ b/src/FOL/IFOL.thy	Wed Mar 04 10:45:52 2009 +0100
@@ -1,5 +1,4 @@
 (*  Title:      FOL/IFOL.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson and Markus Wenzel
 *)
 
@@ -14,9 +13,10 @@
   "~~/src/Tools/IsaPlanner/isand.ML"
   "~~/src/Tools/IsaPlanner/rw_tools.ML"
   "~~/src/Tools/IsaPlanner/rw_inst.ML"
-  "~~/src/Provers/eqsubst.ML"
+  "~~/src/Tools/eqsubst.ML"
   "~~/src/Provers/quantifier1.ML"
-  "~~/src/Provers/project_rule.ML"
+  "~~/src/Tools/intuitionistic.ML"
+  "~~/src/Tools/project_rule.ML"
   "~~/src/Tools/atomize_elim.ML"
   ("fologic.ML")
   ("hypsubstdata.ML")
@@ -610,6 +610,8 @@
 
 subsection {* Intuitionistic Reasoning *}
 
+setup {* Intuitionistic.method_setup "iprover" *}
+
 lemma impE':
   assumes 1: "P --> Q"
     and 2: "Q ==> R"