src/HOL/UNITY/Comp/AllocBase.thy
changeset 13786 ab8f39f48a6f
parent 11194 ea13ff5a26d1
child 13798 4c1a53627500
equal deleted inserted replaced
13785:e2fcd88be55d 13786:ab8f39f48a6f
     4     Copyright   1998  University of Cambridge
     4     Copyright   1998  University of Cambridge
     5 
     5 
     6 Common declarations for Chandy and Charpentier's Allocator
     6 Common declarations for Chandy and Charpentier's Allocator
     7 *)
     7 *)
     8 
     8 
     9 AllocBase = Rename + Follows + 
     9 AllocBase = UNITY_Main + 
    10 
    10 
    11 consts
    11 consts
    12   NbT      :: nat       (*Number of tokens in system*)
    12   NbT      :: nat       (*Number of tokens in system*)
    13   Nclients :: nat       (*Number of clients*)
    13   Nclients :: nat       (*Number of clients*)
    14 
    14