src/HOLCF/IOA/NTP/Correctness.ML
changeset 5068 fb28eaa07e01
parent 4833 2e53109d4bc8
child 5192 704dd3a6d47d
--- a/src/HOLCF/IOA/NTP/Correctness.ML	Mon Jun 22 17:12:27 1998 +0200
+++ b/src/HOLCF/IOA/NTP/Correctness.ML	Mon Jun 22 17:13:09 1998 +0200
@@ -27,7 +27,7 @@
 (* A lemma about restricting the action signature of the implementation
  * to that of the specification.
  ****************************)
-goal Correctness.thy
+Goal
  "a:externals(asig_of(restrict impl_ioa (externals spec_sig))) = \
 \ (case a of                  \
 \     S_msg(m) => True        \
@@ -66,7 +66,7 @@
 
 
 (* Proof of correctness *)
-goalw Correctness.thy [Spec.ioa_def, is_weak_ref_map_def]
+Goalw [Spec.ioa_def, is_weak_ref_map_def]
   "is_weak_ref_map hom (restrict impl_ioa (externals spec_sig)) spec_ioa";
 by (simp_tac (simpset() delsplits [split_if] addsimps 
     [Correctness.hom_def, cancel_restrict, externals_lemma]) 1);