qualified the name "restrict" since Fun.restrict exists too
authorpaulson
Fri, 13 Nov 1998 13:29:50 +0100
changeset 5857 701498a38a76
parent 5856 5fb5a626f3b9
child 5858 beddc19c107a
qualified the name "restrict" since Fun.restrict exists too
src/HOLCF/IOA/NTP/Correctness.ML
--- a/src/HOLCF/IOA/NTP/Correctness.ML	Fri Nov 13 13:29:04 1998 +0100
+++ b/src/HOLCF/IOA/NTP/Correctness.ML	Fri Nov 13 13:29:50 1998 +0100
@@ -28,7 +28,7 @@
  * to that of the specification.
  ****************************)
 Goal
- "a:externals(asig_of(restrict impl_ioa (externals spec_sig))) = \
+ "a:externals(asig_of(Automata.restrict impl_ioa (externals spec_sig))) = \
 \ (case a of                  \
 \     S_msg(m) => True        \
 \   | R_msg(m) => True        \
@@ -67,7 +67,8 @@
 
 (* Proof of correctness *)
 Goalw [Spec.ioa_def, is_weak_ref_map_def]
-  "is_weak_ref_map hom (restrict impl_ioa (externals spec_sig)) spec_ioa";
+  "is_weak_ref_map hom (Automata.restrict impl_ioa (externals spec_sig))  \
+\                  spec_ioa";
 by (simp_tac (simpset() delsplits [split_if] addsimps 
     [Correctness.hom_def, cancel_restrict, externals_lemma]) 1);
 by (rtac conjI 1);