--- a/src/HOL/NanoJava/Decl.thy Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/NanoJava/Decl.thy Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
header "Types, class Declarations, and whole programs"
-theory Decl = Term:
+theory Decl imports Term begin
datatype ty
= NT --{* null type *}