src/HOLCF/Cprod2.ML
changeset 1168 74be52691d62
parent 899 516f9e349a16
child 1267 bca91b4e1710
--- a/src/HOLCF/Cprod2.ML	Thu Jun 29 16:16:24 1995 +0200
+++ b/src/HOLCF/Cprod2.ML	Thu Jun 29 16:28:40 1995 +0200
@@ -9,7 +9,7 @@
 open Cprod2;
 
 qed_goal "less_cprod3a" Cprod2.thy 
-	"p1=<UU,UU> ==> p1 << p2"
+	"p1=(UU,UU) ==> p1 << p2"
  (fn prems =>
 	[
 	(cut_facts_tac prems 1),
@@ -31,7 +31,7 @@
 	]);
 
 qed_goal "less_cprod4a" Cprod2.thy 
-	"<x1,x2> << <UU,UU> ==> x1=UU & x2=UU"
+	"(x1,x2) << (UU,UU) ==> x1=UU & x2=UU"
  (fn prems =>
 	[
 	(cut_facts_tac prems 1),
@@ -40,7 +40,7 @@
 	]);
 
 qed_goal "less_cprod4b" Cprod2.thy 
-	"p << <UU,UU> ==> p = <UU,UU>"
+	"p << (UU,UU) ==> p = (UU,UU)"
 (fn prems =>
 	[
 	(cut_facts_tac prems 1),
@@ -49,7 +49,7 @@
 	]);
 
 qed_goal "less_cprod4c" Cprod2.thy
- " <xa,ya> << <x,y> ==> xa<<x & ya << y"
+ " (xa,ya) << (x,y) ==> xa<<x & ya << y"
 (fn prems =>
 	[
 	(cut_facts_tac prems 1),
@@ -62,7 +62,7 @@
 (* type cprod is pointed                                                    *)
 (* ------------------------------------------------------------------------ *)
 
-qed_goal "minimal_cprod" Cprod2.thy  "<UU,UU><<p"
+qed_goal "minimal_cprod" Cprod2.thy  "(UU,UU)<<p"
 (fn prems =>
 	[
 	(rtac less_cprod3a 1),
@@ -94,7 +94,7 @@
 	]);
 
 qed_goal "monofun_pair" Cprod2.thy 
- "[|x1<<x2; y1<<y2|] ==> <x1,y1> << <x2,y2>"
+ "[|x1<<x2; y1<<y2|] ==> (x1,y1) << (x2,y2)"
  (fn prems =>
 	[
 	(cut_facts_tac prems 1),
@@ -140,7 +140,7 @@
 
 qed_goal "lub_cprod" Cprod2.thy 
 " is_chain(S) ==> range(S) <<| \
-\   < lub(range(%i.fst(S(i)))),lub(range(%i.snd(S(i))))> "
+\   (lub(range(%i.fst(S i))),lub(range(%i.snd(S i)))) "
  (fn prems =>
 	[
 	(cut_facts_tac prems 1),
@@ -166,9 +166,12 @@
 	]);
 
 val thelub_cprod = (lub_cprod RS thelubI);
-(* "is_chain(?S1) ==> lub(range(?S1)) =                                *)
-(*  <lub(range(%i. fst(?S1(i)))), lub(range(%i. snd(?S1(i))))>"        *)
+(*
+"is_chain ?S1 ==>
+ lub (range ?S1) =
+ (lub (range (%i. fst (?S1 i))), lub (range (%i. snd (?S1 i))))" : thm
 
+*)
 
 qed_goal "cpo_cprod" Cprod2.thy 
 	"is_chain(S::nat=>'a*'b)==>? x.range(S)<<| x"
@@ -179,3 +182,4 @@
 	(etac lub_cprod 1)
 	]);
 
+