src/HOL/Bali/State.thy
changeset 80768 c7723cc15de8
parent 77645 7edbb16bc60f
child 80914 d97fdabd9e2b
equal deleted inserted replaced
80767:079fe4292526 80768:c7723cc15de8
   132 
   132 
   133 type_synonym oref = "loc + qtname"         \<comment> \<open>generalized object reference\<close>
   133 type_synonym oref = "loc + qtname"         \<comment> \<open>generalized object reference\<close>
   134 syntax
   134 syntax
   135   Heap  :: "loc   \<Rightarrow> oref"
   135   Heap  :: "loc   \<Rightarrow> oref"
   136   Stat  :: "qtname \<Rightarrow> oref"
   136   Stat  :: "qtname \<Rightarrow> oref"
       
   137 
       
   138 syntax_consts
       
   139   Heap == Inl and
       
   140   Stat == Inr
   137 
   141 
   138 translations
   142 translations
   139   "Heap" => "CONST Inl"
   143   "Heap" => "CONST Inl"
   140   "Stat" => "CONST Inr"
   144   "Stat" => "CONST Inr"
   141   (type) "oref" <= (type) "loc + qtname"
   145   (type) "oref" <= (type) "loc + qtname"