src/HOLCF/Sprod3.ML
changeset 1043 ffa68eb2730b
parent 892 d0dc8d057929
child 1168 74be52691d62
--- a/src/HOLCF/Sprod3.ML	Thu Apr 13 14:18:22 1995 +0200
+++ b/src/HOLCF/Sprod3.ML	Thu Apr 13 14:25:45 1995 +0200
@@ -31,10 +31,6 @@
 	(asm_simp_tac Sprod_ss 1),
 	(rtac sym 1),
 	(rtac lub_chain_maxelem 1),
-	(rtac (monofun_Issnd RS ch2ch_monofun) 1),
-	(rtac ch2ch_fun 1),
-	(rtac (monofun_Ispair1 RS ch2ch_monofun) 1),
-	(atac 1),
 	(res_inst_tac [("P","%j.~Y(j)=UU")] exE 1),
 	(rtac (notall2ex RS iffD1) 1),
 	(res_inst_tac [("Q","lub(range(Y)) = UU")] contrapos 1),
@@ -53,7 +49,6 @@
 	(rtac minimal 1)
 	]);
 
-
 qed_goal "sprod3_lemma2" Sprod3.thy 
 "[| is_chain(Y); ~ x = UU; lub(range(Y)) = UU |] ==>\
 \   Ispair(lub(range(Y)),x) =\
@@ -127,15 +122,12 @@
 \         Ispair(x,lub(range(Y))) =\
 \         Ispair(lub(range(%i. Isfst(Ispair(x,Y(i))))),\
 \                lub(range(%i. Issnd(Ispair(x,Y(i))))))"
-(fn prems =>
+ (fn prems =>
 	[
 	(cut_facts_tac prems 1),
 	(res_inst_tac [("f1","Ispair")] (arg_cong RS cong) 1),
 	(rtac sym 1),
 	(rtac lub_chain_maxelem 1),
-	(rtac (monofun_Isfst RS ch2ch_monofun) 1),
-	(rtac (monofun_Ispair2 RS ch2ch_monofun) 1),
-	(atac 1),
 	(res_inst_tac [("P","%j.~Y(j)=UU")] exE 1),
 	(rtac (notall2ex RS iffD1) 1),
 	(res_inst_tac [("Q","lub(range(Y)) = UU")] contrapos 1),