src/ZF/UNITY/AllocBase.thy
changeset 16417 9bc16273c2d4
parent 14095 a1ba833d6b61
child 24892 c663e675e177
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     5 
     5 
     6 *)
     6 *)
     7 
     7 
     8 header{*Common declarations for Chandy and Charpentier's Allocator*}
     8 header{*Common declarations for Chandy and Charpentier's Allocator*}
     9 
     9 
    10 theory AllocBase = Follows + MultisetSum + Guar:
    10 theory AllocBase imports Follows MultisetSum Guar begin
    11 
    11 
    12 consts
    12 consts
    13   tokbag   :: i  (* tokbags could be multisets...or any ordered type?*)
    13   tokbag   :: i  (* tokbags could be multisets...or any ordered type?*)
    14   NbT      :: i  (* Number of tokens in system *)
    14   NbT      :: i  (* Number of tokens in system *)
    15   Nclients :: i  (* Number of clients *)
    15   Nclients :: i  (* Number of clients *)