src/ZF/AC/AC_Equiv.ML
changeset 12667 7e6eaaa125f2
parent 11317 7f9e4c389318
--- a/src/ZF/AC/AC_Equiv.ML	Tue Jan 08 15:39:47 2002 +0100
+++ b/src/ZF/AC/AC_Equiv.ML	Tue Jan 08 16:09:09 2002 +0100
@@ -26,7 +26,7 @@
 
 (* used in \\<in> AC10-AC15.ML AC16WO4.ML WO6WO1.ML *)
 (*I don't know where to put this one.*)
-goal Cardinal.thy
+Goal
      "!!m A B. [| A lepoll succ(m); B \\<subseteq> A; B\\<noteq>0 |] ==> A-B lepoll m";
 by (rtac not_emptyE 1 THEN (assume_tac 1));
 by (ftac singleton_subsetI 1);
@@ -65,7 +65,7 @@
 qed "ordertype_Int";
 
 (* used only in AC16_lemmas.ML *)
-goalw CardinalArith.thy [InfCard_def]
+Goalw [InfCard_def]
         "!!i. [| ~Finite(i); Card(i) |] ==> InfCard(i)";
 by (asm_simp_tac (simpset() addsimps [Card_is_Ord RS nat_le_infinite_Ord]) 1);
 qed "Inf_Card_is_InfCard";