src/HOL/IOA/NTP/Receiver.ML
changeset 1266 3ae9fe3c0f68
parent 1051 4fcd0638e61d
child 1328 9a449a91425d
--- a/src/HOL/IOA/NTP/Receiver.ML	Wed Oct 04 13:11:57 1995 +0100
+++ b/src/HOL/IOA/NTP/Receiver.ML	Wed Oct 04 13:12:14 1995 +0100
@@ -15,9 +15,8 @@
 \ 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);
+  by(simp_tac (!simpset addsimps (Receiver.receiver_asig_def :: actions_def :: 
+                                  asig_projections @ set_lemmas)) 1);
 qed "in_receiver_asig";
 
 val receiver_projections =