src/HOL/MicroJava/J/Value.thy
changeset 12338 de0f4a63baa5
parent 11908 82f68fd05094
child 12517 360e3215f029
equal deleted inserted replaced
12337:7c6a970f0808 12338:de0f4a63baa5
     7 header "Java Values"
     7 header "Java Values"
     8 
     8 
     9 theory Value = Type:
     9 theory Value = Type:
    10 
    10 
    11 typedecl loc (* locations, i.e. abstract references on objects *)
    11 typedecl loc (* locations, i.e. abstract references on objects *)
    12 arities loc :: "term"
       
    13 
    12 
    14 datatype val
    13 datatype val
    15   = Unit        (* dummy result value of void methods *)
    14   = Unit        (* dummy result value of void methods *)
    16   | Null        (* null reference *)
    15   | Null        (* null reference *)
    17   | Bool bool   (* Boolean value *)
    16   | Bool bool   (* Boolean value *)