src/HOL/MicroJava/Comp/TranslCompTp.thy
changeset 15481 fc075ae929e4
parent 14981 e73f8140af78
child 32960 69916a850301
--- a/src/HOL/MicroJava/Comp/TranslCompTp.thy	Sun Jan 30 20:48:50 2005 +0100
+++ b/src/HOL/MicroJava/Comp/TranslCompTp.thy	Tue Feb 01 18:01:57 2005 +0100
@@ -3,7 +3,10 @@
     Author:     Martin Strecker
 *)
 
-theory TranslCompTp =  JVMType + Index:
+theory TranslCompTp
+imports Index "../BV/JVMType"
+begin
+
 
 
 (**********************************************************************)