src/HOLCF/Discrete1.ML
changeset 5068 fb28eaa07e01
parent 4721 c8a8482a8124
child 5192 704dd3a6d47d
--- a/src/HOLCF/Discrete1.ML	Mon Jun 22 17:12:27 1998 +0200
+++ b/src/HOLCF/Discrete1.ML	Mon Jun 22 17:13:09 1998 +0200
@@ -6,12 +6,12 @@
 Proves that 'a discr is a cpo
 *)
 
-goalw thy [less_discr_def] "((x::('a::term)discr) << y) = (x=y)";
+Goalw [less_discr_def] "((x::('a::term)discr) << y) = (x=y)";
 by (rtac refl 1);
 qed "discr_less_eq";
 AddIffs [discr_less_eq];
 
-goalw thy [chain]
+Goalw [chain]
  "!!S::nat=>('a::term)discr. chain S ==> S i = S 0";
 by (nat_ind_tac "i" 1);
 by (rtac refl 1);
@@ -20,13 +20,13 @@
 by (Fast_tac 1);
 qed "discr_chain0";
 
-goal thy
+Goal
  "!!S::nat=>('a::term)discr. chain(S) ==> range(S) = {S 0}";
 by (fast_tac (claset() addEs [discr_chain0]) 1);
 qed "discr_chain_range0";
 Addsimps [discr_chain_range0];
 
-goalw thy [is_lub,is_ub]
+Goalw [is_lub,is_ub]
  "!!S. chain S ==> ? x::('a::term)discr. range(S) <<| x";
 by (Asm_simp_tac 1);
 qed "discr_cpo";