fixed imports path;
authorwenzelm
Fri, 09 Nov 2007 19:37:32 +0100
changeset 25363 fbdfceb8de15
parent 25362 8d06e11a01d1
child 25364 7f012f56efa3
fixed imports path;
src/HOL/MicroJava/BV/JType.thy
--- a/src/HOL/MicroJava/BV/JType.thy	Fri Nov 09 19:37:30 2007 +0100
+++ b/src/HOL/MicroJava/BV/JType.thy	Fri Nov 09 19:37:32 2007 +0100
@@ -6,7 +6,7 @@
 
 header {* \isaheader{The Java Type System as Semilattice} *}
 
-theory JType imports WellForm Err begin
+theory JType imports "../J/WellForm" Err begin
 
 constdefs
   super :: "'a prog \<Rightarrow> cname \<Rightarrow> cname"