src/HOL/MicroJava/J/Decl.thy
changeset 16417 9bc16273c2d4
parent 14134 0fdf5708c7a8
child 18551 be0705186ff5
--- a/src/HOL/MicroJava/J/Decl.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/MicroJava/J/Decl.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* \isaheader{Class Declarations and Programs} *}
 
-theory Decl = Type:
+theory Decl imports Type begin
 
 types 
   fdecl    = "vname \<times> ty"        -- "field declaration, cf. 8.3 (, 9.3)"