src/HOL/MicroJava/J/WellForm.thy
changeset 16417 9bc16273c2d4
parent 15481 fc075ae929e4
child 18447 da548623916a
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4     Copyright   1999 Technische Universitaet Muenchen
     4     Copyright   1999 Technische Universitaet Muenchen
     5 *)
     5 *)
     6 
     6 
     7 header {* \isaheader{Well-formedness of Java programs} *}
     7 header {* \isaheader{Well-formedness of Java programs} *}
     8 
     8 
     9 theory WellForm = TypeRel + SystemClasses:
     9 theory WellForm imports TypeRel SystemClasses begin
    10 
    10 
    11 text {*
    11 text {*
    12 for static checks on expressions and statements, see WellType.
    12 for static checks on expressions and statements, see WellType.
    13 
    13 
    14 \begin{description}
    14 \begin{description}