src/HOL/Bali/DeclConcepts.thy
changeset 16417 9bc16273c2d4
parent 14981 e73f8140af78
child 19564 d3e2f532459a
--- a/src/HOL/Bali/DeclConcepts.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Bali/DeclConcepts.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 header {* Advanced concepts on Java declarations like overriding, inheritance,
 dynamic method lookup*}
 
-theory DeclConcepts = TypeRel:
+theory DeclConcepts imports TypeRel begin
 
 section "access control (cf. 6.6), overriding and hiding (cf. 8.4.6.1)"