src/HOL/UNITY/Comp/Priority.thy
changeset 16417 9bc16273c2d4
parent 16184 80617b8d33c5
child 35416 d8d7d1b785af
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4     Copyright   2001  University of Cambridge
     4     Copyright   2001  University of Cambridge
     5 *)
     5 *)
     6 
     6 
     7 header{*The priority system*}
     7 header{*The priority system*}
     8 
     8 
     9 theory Priority = PriorityAux:
     9 theory Priority imports PriorityAux begin
    10 
    10 
    11 text{*From Charpentier and Chandy,
    11 text{*From Charpentier and Chandy,
    12 Examples of Program Composition Illustrating the Use of Universal Properties
    12 Examples of Program Composition Illustrating the Use of Universal Properties
    13    In J. Rolim (editor), Parallel and Distributed Processing,
    13    In J. Rolim (editor), Parallel and Distributed Processing,
    14    Spriner LNCS 1586 (1999), pages 1215-1227.*}
    14    Spriner LNCS 1586 (1999), pages 1215-1227.*}