src/HOL/HOLCF/IOA/meta_theory/Traces.thy
changeset 62000 8cba509ace9c
parent 61032 b57df8eecad6
child 62001 1f2788fb0b8b
equal deleted inserted replaced
61999:89291b5d0ede 62000:8cba509ace9c
   153                       then ~Enabled A W (laststate ex)
   153                       then ~Enabled A W (laststate ex)
   154                       else is_wfair A W ex"
   154                       else is_wfair A W ex"
   155 
   155 
   156 is_wfair_def:
   156 is_wfair_def:
   157   "is_wfair A W ex == (inf_often (%x. fst x:W) (snd ex)
   157   "is_wfair A W ex == (inf_often (%x. fst x:W) (snd ex)
   158                      | inf_often (%x.~Enabled A W (snd x)) (snd ex))"
   158                      | inf_often (%x. ~ Enabled A W (snd x)) (snd ex))"
   159 
   159 
   160 sfair_ex_def:
   160 sfair_ex_def:
   161   "sfair_ex A ex == ! W : sfair_of A.
   161   "sfair_ex A ex == ! W : sfair_of A.
   162                       if   Finite (snd ex)
   162                       if   Finite (snd ex)
   163                       then ~Enabled A W (laststate ex)
   163                       then ~Enabled A W (laststate ex)