src/HOL/MicroJava/Comp/TypeInf.thy
changeset 17778 93d7e524417a
parent 16417 9bc16273c2d4
child 35416 d8d7d1b785af
--- a/src/HOL/MicroJava/Comp/TypeInf.thy	Fri Oct 07 18:49:20 2005 +0200
+++ b/src/HOL/MicroJava/Comp/TypeInf.thy	Fri Oct 07 20:41:10 2005 +0200
@@ -4,7 +4,9 @@
 *)
 
 (* Exact position in theory hierarchy still to be determined *)
-theory TypeInf imports  WellType begin
+theory TypeInf
+imports "../J/WellType"
+begin