IOA/example/Receiver.ML
changeset 252 a4dc62a46ee4
parent 251 f04b33ce250f
child 253 132634d24019
--- a/IOA/example/Receiver.ML	Tue Oct 24 14:59:17 1995 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,30 +0,0 @@
-(*  Title:      HOL/IOA/example/Receiver.ML
-    ID:         $Id$
-    Author:     Tobias Nipkow & Konrad Slind
-    Copyright   1994  TU Muenchen
-*)
-
-goal Receiver.thy
- "S_msg(m) ~: actions(receiver_asig)      &   \
-\ R_msg(m) : actions(receiver_asig)       &   \
-\ S_pkt(pkt) ~: actions(receiver_asig) &   \
-\ R_pkt(pkt) : actions(receiver_asig)  &   \
-\ S_ack(b) : actions(receiver_asig)    &   \
-\ R_ack(b) ~: actions(receiver_asig)   &   \
-\ C_m_s ~: actions(receiver_asig)         &   \
-\ C_m_r : actions(receiver_asig)          &   \
-\ C_r_s ~: actions(receiver_asig)         &   \
-\ C_r_r(m) : actions(receiver_asig)";
-  by(simp_tac (action_ss addsimps 
-               (Receiver.receiver_asig_def :: actions_def :: 
-                asig_projections @ set_lemmas)) 1);
-qed "in_receiver_asig";
-
-val receiver_projections = 
-   [Receiver.rq_def,
-    Receiver.rsent_def,
-    Receiver.rrcvd_def,
-    Receiver.rbit_def,
-    Receiver.rsending_def];
-
-