src/HOL/TLA/Memory/MIParameters.thy
changeset 5184 9b8547a9496a
parent 3807 82a99b090d9d
child 11703 6e5de8d4290a
equal deleted inserted replaced
5183:89f162de39cf 5184:9b8547a9496a
     7     Logic Image: TLA
     7     Logic Image: TLA
     8 
     8 
     9     RPC-Memory example: Parameters of the memory implementation.
     9     RPC-Memory example: Parameters of the memory implementation.
    10 *)
    10 *)
    11 
    11 
    12 MIParameters = Arith +
    12 MIParameters = Datatype +
    13 
    13 
    14 datatype  histState  =  histA | histB
    14 datatype  histState  =  histA | histB
    15 
    15 
    16 end
    16 end
    17 
    17