src/HOL/UNITY/WFair.thy
changeset 16417 9bc16273c2d4
parent 15045 d59f7e2e18d3
child 19769 c40ce2de2020
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     8 From Misra, "A Logic for Concurrent Programming", 1994
     8 From Misra, "A Logic for Concurrent Programming", 1994
     9 *)
     9 *)
    10 
    10 
    11 header{*Progress*}
    11 header{*Progress*}
    12 
    12 
    13 theory WFair = UNITY:
    13 theory WFair imports UNITY begin
    14 
    14 
    15 text{*The original version of this theory was based on weak fairness.  (Thus,
    15 text{*The original version of this theory was based on weak fairness.  (Thus,
    16 the entire UNITY development embodied this assumption, until February 2003.)
    16 the entire UNITY development embodied this assumption, until February 2003.)
    17 Weak fairness states that if a command is enabled continuously, then it is
    17 Weak fairness states that if a command is enabled continuously, then it is
    18 eventually executed.  Ernie Cohen suggested that I instead adopt unconditional
    18 eventually executed.  Ernie Cohen suggested that I instead adopt unconditional