src/HOL/HOL.thy
changeset 28952 15a4b2cf8c34
parent 28856 5e009a80fe6d
child 29105 8f38bf68d42e
--- a/src/HOL/HOL.thy	Wed Dec 03 09:53:58 2008 +0100
+++ b/src/HOL/HOL.thy	Wed Dec 03 15:58:44 2008 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/HOL.thy
-    ID:         $Id$
     Author:     Tobias Nipkow, Markus Wenzel, and Larry Paulson
 *)
 
@@ -8,7 +7,7 @@
 theory HOL
 imports Pure
 uses
-  ("hologic.ML")
+  ("Tools/hologic.ML")
   "~~/src/Tools/IsaPlanner/zipper.ML"
   "~~/src/Tools/IsaPlanner/isand.ML"
   "~~/src/Tools/IsaPlanner/rw_tools.ML"
@@ -22,7 +21,7 @@
   "~~/src/Provers/coherent.ML"
   "~~/src/Provers/eqsubst.ML"
   "~~/src/Provers/quantifier1.ML"
-  ("simpdata.ML")
+  ("Tools/simpdata.ML")
   "~~/src/Tools/random_word.ML"
   "~~/src/Tools/atomize_elim.ML"
   "~~/src/Tools/induct.ML"
@@ -801,7 +800,7 @@
   and [sym] = sym not_sym
   and [Pure.elim?] = iffD1 iffD2 impE
 
-use "hologic.ML"
+use "Tools/hologic.ML"
 
 
 subsubsection {* Atomizing meta-level connectives *}
@@ -1285,7 +1284,7 @@
   "(\<exists>x y. P x y) = (\<exists>y x. P x y)"
   by blast
 
-use "simpdata.ML"
+use "Tools/simpdata.ML"
 ML {* open Simpdata *}
 
 setup {*