156
|
1 |
goal Receiver.thy
|
|
2 |
"S_msg(m) ~: actions(receiver_asig) & \
|
|
3 |
\ R_msg(m) : actions(receiver_asig) & \
|
|
4 |
\ S_pkt(pkt) ~: actions(receiver_asig) & \
|
|
5 |
\ R_pkt(pkt) : actions(receiver_asig) & \
|
|
6 |
\ S_ack(b) : actions(receiver_asig) & \
|
|
7 |
\ R_ack(b) ~: actions(receiver_asig) & \
|
|
8 |
\ C_m_s ~: actions(receiver_asig) & \
|
|
9 |
\ C_m_r : actions(receiver_asig) & \
|
|
10 |
\ C_r_s ~: actions(receiver_asig) & \
|
|
11 |
\ C_r_r(m) : actions(receiver_asig)";
|
|
12 |
by(simp_tac (action_ss addsimps
|
|
13 |
(Receiver.receiver_asig_def :: actions_def ::
|
|
14 |
asig_projections_def :: set_lemmas)) 1);
|
|
15 |
val in_receiver_asig = result();
|
|
16 |
|
|
17 |
val receiver_projections =
|
|
18 |
[Receiver.rq_def,
|
|
19 |
Receiver.rsent_def,
|
|
20 |
Receiver.rrcvd_def,
|
|
21 |
Receiver.rbit_def,
|
|
22 |
Receiver.rsending_def];
|
|
23 |
|
|
24 |
|