| changeset 16417 | 9bc16273c2d4 |
| parent 15481 | fc075ae929e4 |
| child 18447 | da548623916a |
--- a/src/HOL/MicroJava/J/WellForm.thy Fri Jun 17 11:35:35 2005 +0200 +++ b/src/HOL/MicroJava/J/WellForm.thy Fri Jun 17 16:12:49 2005 +0200 @@ -6,7 +6,7 @@ header {* \isaheader{Well-formedness of Java programs} *} -theory WellForm = TypeRel + SystemClasses: +theory WellForm imports TypeRel SystemClasses begin text {* for static checks on expressions and statements, see WellType.