src/HOLCF/Cfun3.ML
changeset 961 932784dfa671
parent 892 d0dc8d057929
child 1168 74be52691d62
--- a/src/HOLCF/Cfun3.ML	Thu Mar 16 00:00:30 1995 +0100
+++ b/src/HOLCF/Cfun3.ML	Fri Mar 17 15:35:09 1995 +0100
@@ -205,7 +205,7 @@
 (* function application _[_]  is strict in its first arguments              *)
 (* ------------------------------------------------------------------------ *)
 
-qed_goal "strict_fapp1" Cfun3.thy "UU[x] = UU"
+qed_goal "strict_fapp1" Cfun3.thy "(UU::'a->'b)[x] = (UU::'b)"
  (fn prems =>
 	[
 	(rtac (inst_cfun_pcpo RS ssubst) 1),
@@ -221,7 +221,7 @@
 (* ------------------------------------------------------------------------ *)
 
 qed_goalw "Istrictify1" Cfun3.thy [Istrictify_def]
-	"Istrictify(f)(UU)=UU"
+	"Istrictify(f)(UU)= (UU)"
  (fn prems =>
 	[
 	(rtac select_equality 1),
@@ -305,12 +305,12 @@
 	(rtac (refl RS allI) 1)
 	]);
 
-qed_goal "contlub_Istrictify2" Cfun3.thy "contlub(Istrictify(f))"
+qed_goal "contlub_Istrictify2" Cfun3.thy "contlub(Istrictify(f::'a -> 'b))"
  (fn prems =>
 	[
 	(rtac contlubI 1),
 	(strip_tac 1),
-	(res_inst_tac [("Q","lub(range(Y))=UU")] classical2 1),
+	(res_inst_tac [("Q","lub(range(Y))=(UU::'a)")] classical2 1),
 	(res_inst_tac [("t","lub(range(Y))")] subst 1),
 	(rtac sym 1),
 	(atac 1),
@@ -318,7 +318,7 @@
 	(rtac sym 1),
 	(rtac chain_UU_I_inverse 1),
 	(strip_tac 1),
-	(res_inst_tac [("t","Y(i)"),("s","UU")] subst 1),
+	(res_inst_tac [("t","Y(i)"),("s","UU::'a")] subst 1),
 	(rtac sym 1),
 	(rtac (chain_UU_I RS spec) 1),
 	(atac 1),
@@ -347,7 +347,7 @@
 	]);
 
 
-val contX_Istrictify1 =	(contlub_Istrictify1 RS 
+val contX_Istrictify1 = (contlub_Istrictify1 RS 
 	(monofun_Istrictify1 RS monocontlub2contX)); 
 
 val contX_Istrictify2 = (contlub_Istrictify2 RS