src/ZF/ex/Ramsey.ML
changeset 760 f0200e91b272
parent 694 c7d592f6312a
child 782 200a16083201
--- a/src/ZF/ex/Ramsey.ML	Wed Dec 07 12:34:47 1994 +0100
+++ b/src/ZF/ex/Ramsey.ML	Wed Dec 07 13:12:04 1994 +0100
@@ -44,7 +44,7 @@
 
 goalw Ramsey.thy [Atleast_def, inj_def, Pi_def, function_def] "Atleast(0,A)";
 by (fast_tac ZF_cs 1);
-val Atleast0 = result();
+qed "Atleast0";
 
 val [major] = goalw Ramsey.thy [Atleast_def]
     "Atleast(succ(m),A) ==> EX x:A. Atleast(m, A-{x})";
@@ -54,7 +54,7 @@
 by (rtac succI1 2);
 by (rtac exI 1);
 by (etac inj_succ_restrict 1);
-val Atleast_succD = result();
+qed "Atleast_succD";
 
 val major::prems = goalw Ramsey.thy [Atleast_def]
     "[| Atleast(n,A);  A<=B |] ==> Atleast(n,B)";
@@ -62,7 +62,7 @@
 by (rtac exI 1);
 by (etac inj_weaken_type 1);
 by (resolve_tac prems 1);
-val Atleast_superset = result();
+qed "Atleast_superset";
 
 val prems = goalw Ramsey.thy [Atleast_def,succ_def]
     "[| Atleast(m,B);  b~: B |] ==> Atleast(succ(m), cons(b,B))";
@@ -72,7 +72,7 @@
 by (etac inj_extend 1);
 by (rtac mem_not_refl 1);
 by (assume_tac 1);
-val Atleast_succI = result();
+qed "Atleast_succI";
 
 val prems = goal Ramsey.thy
     "[| Atleast(m, B-{x});  x: B |] ==> Atleast(succ(m), B)";
@@ -80,7 +80,7 @@
 by (etac (Atleast_succI RS Atleast_superset) 1);
 by (fast_tac ZF_cs 1);
 by (fast_tac ZF_cs 1);
-val Atleast_Diff_succI = result();
+qed "Atleast_Diff_succI";
 
 (*** Main Cardinality Lemma ***)