src/HOL/MicroJava/J/State.thy
changeset 16417 9bc16273c2d4
parent 14174 f3cafd2929d5
child 24783 5a3e336a2e37
     1.1 --- a/src/HOL/MicroJava/J/State.thy	Fri Jun 17 11:35:35 2005 +0200
     1.2 +++ b/src/HOL/MicroJava/J/State.thy	Fri Jun 17 16:12:49 2005 +0200
     1.3 @@ -6,7 +6,7 @@
     1.4  
     1.5  header {* \isaheader{Program State} *}
     1.6  
     1.7 -theory State = TypeRel + Value:
     1.8 +theory State imports TypeRel Value begin
     1.9  
    1.10  types 
    1.11    fields_ = "(vname \<times> cname \<rightharpoonup> val)"  -- "field name, defining class, value"