src/HOL/NanoJava/State.thy
changeset 58249 180f1b3508ed
parent 55466 786edc984c98
child 58310 91ea607a34d8
equal deleted inserted replaced
58248:25af24e1f37b 58249:180f1b3508ed
    11  "body \<equiv> \<lambda>(C,m). bdy (the (method C m))"
    11  "body \<equiv> \<lambda>(C,m). bdy (the (method C m))"
    12 
    12 
    13 text {* Locations, i.e.\ abstract references to objects *}
    13 text {* Locations, i.e.\ abstract references to objects *}
    14 typedecl loc 
    14 typedecl loc 
    15 
    15 
    16 datatype val
    16 datatype_new val
    17   = Null        --{* null reference *}
    17   = Null        --{* null reference *}
    18   | Addr loc    --{* address, i.e. location of object *}
    18   | Addr loc    --{* address, i.e. location of object *}
    19 
    19 
    20 type_synonym fields
    20 type_synonym fields
    21         = "(fname \<rightharpoonup> val)"
    21         = "(fname \<rightharpoonup> val)"