168
|
1 |
(* Title: HOL/IOA/example/Receiver.ML
|
|
2 |
ID: $Id$
|
|
3 |
Author: Tobias Nipkow & Konrad Slind
|
|
4 |
Copyright 1994 TU Muenchen
|
|
5 |
*)
|
|
6 |
|
156
|
7 |
goal Receiver.thy
|
|
8 |
"S_msg(m) ~: actions(receiver_asig) & \
|
|
9 |
\ R_msg(m) : actions(receiver_asig) & \
|
|
10 |
\ S_pkt(pkt) ~: actions(receiver_asig) & \
|
|
11 |
\ R_pkt(pkt) : actions(receiver_asig) & \
|
|
12 |
\ S_ack(b) : actions(receiver_asig) & \
|
|
13 |
\ R_ack(b) ~: actions(receiver_asig) & \
|
|
14 |
\ C_m_s ~: actions(receiver_asig) & \
|
|
15 |
\ C_m_r : actions(receiver_asig) & \
|
|
16 |
\ C_r_s ~: actions(receiver_asig) & \
|
|
17 |
\ C_r_r(m) : actions(receiver_asig)";
|
|
18 |
by(simp_tac (action_ss addsimps
|
|
19 |
(Receiver.receiver_asig_def :: actions_def ::
|
168
|
20 |
asig_projections @ set_lemmas)) 1);
|
156
|
21 |
val in_receiver_asig = result();
|
|
22 |
|
|
23 |
val receiver_projections =
|
|
24 |
[Receiver.rq_def,
|
|
25 |
Receiver.rsent_def,
|
|
26 |
Receiver.rrcvd_def,
|
|
27 |
Receiver.rbit_def,
|
|
28 |
Receiver.rsending_def];
|
|
29 |
|
|
30 |
|