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