IOA/example/Sender.ML
changeset 168 44ff2275d44f
parent 156 fd1be45b64bf
child 171 16c4ea954511
--- a/IOA/example/Sender.ML	Wed Nov 09 19:50:36 1994 +0100
+++ b/IOA/example/Sender.ML	Wed Nov 09 19:51:09 1994 +0100
@@ -1,3 +1,9 @@
+(*  Title:      HOL/IOA/example/Sender.ML
+    ID:         $Id$
+    Author:     Tobias Nipkow & Konrad Slind
+    Copyright   1994  TU Muenchen
+*)
+
 goal Sender.thy
  "S_msg(m) : actions(sender_asig)       &   \
 \ R_msg(m) ~: actions(sender_asig)      &   \
@@ -11,7 +17,7 @@
 \ C_r_r(m) ~: actions(sender_asig)";
 by(simp_tac (action_ss addsimps 
              (Sender.sender_asig_def :: actions_def :: 
-              asig_projections_def :: set_lemmas)) 1);
+              asig_projections @ set_lemmas)) 1);
 val in_sender_asig = result();
 
 val sender_projections =