corrected problems with changed binding power of ::.
authornipkow
Mon, 10 Oct 1994 18:09:58 +0100
changeset 628 bb3f87f9cafe
parent 627 e685b5411617
child 629 c97f5a7cf763
corrected problems with changed binding power of ::.
src/HOLCF/Fix.ML
src/HOLCF/Pcpo.thy
--- a/src/HOLCF/Fix.ML	Mon Oct 10 12:57:23 1994 +0100
+++ b/src/HOLCF/Fix.ML	Mon Oct 10 18:09:58 1994 +0100
@@ -693,17 +693,17 @@
 (* ------------------------------------------------------------------------- *)
 
 val flat_codom = prove_goalw Fix.thy [flat_def]
-"[|flat(y::'b);f[x::'a]=(c::'b)|] ==> f[UU::'a]=UU::'b | (!z.f[z::'a]=c)"
+"[|flat(y::'b);f[x::'a]=(c::'b)|] ==> f[UU::'a]=(UU::'b) | (!z.f[z::'a]=c)"
  (fn prems =>
 	[
 	(cut_facts_tac prems 1),
-	(res_inst_tac [("Q","f[x::'a]=UU::'b")] classical2 1),
+	(res_inst_tac [("Q","f[x::'a]=(UU::'b)")] classical2 1),
 	(rtac disjI1 1),
 	(rtac UU_I 1),
 	(res_inst_tac [("s","f[x]"),("t","UU::'b")] subst 1),
 	(atac 1),
 	(rtac (minimal RS monofun_cfun_arg) 1),
-	(res_inst_tac [("Q","f[UU::'a]=UU::'b")] classical2 1),
+	(res_inst_tac [("Q","f[UU::'a]=(UU::'b)")] classical2 1),
 	(etac disjI1 1),
 	(rtac disjI2 1),
 	(rtac allI 1),
--- a/src/HOLCF/Pcpo.thy	Mon Oct 10 12:57:23 1994 +0100
+++ b/src/HOLCF/Pcpo.thy	Mon Oct 10 18:09:58 1994 +0100
@@ -8,7 +8,7 @@
 rules
 
 minimal	"UU << x"	
-cpo	"is_chain(S) ==> ? x. range(S) <<| x::('a::pcpo)" 
+cpo	"is_chain(S) ==> ? x. range(S) <<| (x::'a::pcpo)" 
 
 inst_void_pcpo	"(UU::void) = UU_void"