src/HOL/IOA/ABP/Receiver.thy
changeset 1476 608483c2122a
parent 1376 92f83b9d17e1
equal deleted inserted replaced
1475:7f5a4cd08209 1476:608483c2122a
    39       case fst(snd(tr))                                                 
    39       case fst(snd(tr))                                                 
    40       of   
    40       of   
    41       Next    =>  False |     
    41       Next    =>  False |     
    42       S_msg(m) => False |                                               
    42       S_msg(m) => False |                                               
    43       R_msg(m) => (rq(s) ~= [])  &                                     
    43       R_msg(m) => (rq(s) ~= [])  &                                     
    44 		   m = hd(rq(s))  &                             
    44                    m = hd(rq(s))  &                             
    45 		   rq(t) = tl(rq(s))   &                              
    45                    rq(t) = tl(rq(s))   &                              
    46                   rbit(t)=rbit(s)  |                                 
    46                   rbit(t)=rbit(s)  |                                 
    47       S_pkt(pkt) => False |                                          
    47       S_pkt(pkt) => False |                                          
    48       R_pkt(pkt) => if (hdr(pkt) ~= rbit(s))&rq(s)=[] then            
    48       R_pkt(pkt) => if (hdr(pkt) ~= rbit(s))&rq(s)=[] then            
    49 		         rq(t) = (rq(s)@[msg(pkt)]) &rbit(t) = (~rbit(s)) else  
    49                          rq(t) = (rq(s)@[msg(pkt)]) &rbit(t) = (~rbit(s)) else  
    50 		         rq(t) =rq(s) & rbit(t)=rbit(s)  |   
    50                          rq(t) =rq(s) & rbit(t)=rbit(s)  |   
    51       S_ack(b) => b = rbit(s)                        &               
    51       S_ack(b) => b = rbit(s)                        &               
    52                       rq(t) = rq(s)                    &             
    52                       rq(t) = rq(s)                    &             
    53                       rbit(t)=rbit(s) |                              
    53                       rbit(t)=rbit(s) |                              
    54       R_ack(b) => False}"
    54       R_ack(b) => False}"
    55 
    55