src/HOL/MicroJava/J/Conform.thy
changeset 16417 9bc16273c2d4
parent 14174 f3cafd2929d5
child 24783 5a3e336a2e37
--- a/src/HOL/MicroJava/J/Conform.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/MicroJava/J/Conform.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* \isaheader{Conformity Relations for Type Soundness Proof} *}
 
-theory Conform = State + WellType + Exceptions:
+theory Conform imports State WellType Exceptions begin
 
 types 'c env_ = "'c prog \<times> (vname \<rightharpoonup> ty)"  -- "same as @{text env} of @{text WellType.thy}"