src/HOL/IMP/Denotation.ML
changeset 5069 3ea049f7979d
parent 4477 b3e5857d8d99
child 5117 7b5efef2ca74
--- a/src/HOL/IMP/Denotation.ML	Mon Jun 22 17:13:09 1998 +0200
+++ b/src/HOL/IMP/Denotation.ML	Mon Jun 22 17:26:46 1998 +0200
@@ -14,7 +14,7 @@
      (fn _ => [Fast_tac 1]);
 
 
-goal Denotation.thy "C(WHILE b DO c) = C(IF b THEN c;WHILE b DO c ELSE SKIP)";
+Goal "C(WHILE b DO c) = C(IF b THEN c;WHILE b DO c ELSE SKIP)";
 by (Simp_tac 1);
 by (EVERY[stac (Gamma_mono RS lfp_Tarski) 1,
           stac (Gamma_def RS meta_eq_to_obj_eq RS fun_cong) 1,
@@ -25,7 +25,7 @@
 
 (* Operational Semantics implies Denotational Semantics *)
 
-goal Denotation.thy "!!c s t. <c,s> -c-> t ==> (s,t) : C(c)";
+Goal "!!c s t. <c,s> -c-> t ==> (s,t) : C(c)";
 
 (* start with rule induction *)
 by (etac evalc.induct 1);
@@ -41,7 +41,7 @@
 
 (* Denotational Semantics implies Operational Semantics *)
 
-goal Denotation.thy "!s t. (s,t):C(c) --> <c,s> -c-> t";
+Goal "!s t. (s,t):C(c) --> <c,s> -c-> t";
 by (com.induct_tac "c" 1);
 
 by (ALLGOALS Full_simp_tac);
@@ -58,6 +58,6 @@
 
 (**** Proof of Equivalence ****)
 
-goal Denotation.thy "(s,t) : C(c)  =  (<c,s> -c-> t)";
+Goal "(s,t) : C(c)  =  (<c,s> -c-> t)";
 by (fast_tac (claset() addEs [com2] addDs [com1]) 1);
 qed "denotational_is_natural";