--- a/IOA/example/Receiver.ML Wed Nov 09 19:50:36 1994 +0100
+++ b/IOA/example/Receiver.ML Wed Nov 09 19:51:09 1994 +0100
@@ -1,3 +1,9 @@
+(* 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) & \
@@ -11,7 +17,7 @@
\ C_r_r(m) : actions(receiver_asig)";
by(simp_tac (action_ss addsimps
(Receiver.receiver_asig_def :: actions_def ::
- asig_projections_def :: set_lemmas)) 1);
+ asig_projections @ set_lemmas)) 1);
val in_receiver_asig = result();
val receiver_projections =