src/ZF/ex/misc.ML
changeset 38 4433428596f9
parent 16 0b033d50ca1c
child 434 89d45187f04d
--- a/src/ZF/ex/misc.ML	Thu Oct 07 10:48:16 1993 +0100
+++ b/src/ZF/ex/misc.ML	Thu Oct 07 11:47:50 1993 +0100
@@ -26,18 +26,18 @@
   addSEs [CollectE, equalityCE];
 
 (*The search is undirected and similar proof attempts fail*)
-goal ZF.thy "ALL f: A->Pow(A). EX S: Pow(A). ALL x:A. ~ f`x = S";
+goal ZF.thy "ALL f: A->Pow(A). EX S: Pow(A). ALL x:A. f`x ~= S";
 by (best_tac cantor_cs 1);
 result();
 
-(*This form displays the diagonal term, {x: A . ~ x: f`x} *)
+(*This form displays the diagonal term, {x: A . x ~: f`x} *)
 val [prem] = goal ZF.thy
-    "f: A->Pow(A) ==> (ALL x:A. ~ f`x = ?S) & ?S: Pow(A)";
+    "f: A->Pow(A) ==> (ALL x:A. f`x ~= ?S) & ?S: Pow(A)";
 by (best_tac cantor_cs 1);
 result();
 
 (*yet another version...*)
-goalw Perm.thy [surj_def] "~ f : surj(A,Pow(A))";
+goalw Perm.thy [surj_def] "f ~: surj(A,Pow(A))";
 by (safe_tac ZF_cs);
 by (etac ballE 1);
 by (best_tac (cantor_cs addSEs [bexE]) 1);