src/HOL/Set.ML
changeset 2031 03a843f0f447
parent 2024 909153d8318f
child 2499 0bc87b063447
--- a/src/HOL/Set.ML	Thu Sep 26 11:11:22 1996 +0200
+++ b/src/HOL/Set.ML	Thu Sep 26 12:47:47 1996 +0200
@@ -11,7 +11,7 @@
 section "Relating predicates and sets";
 
 val [prem] = goal Set.thy "P(a) ==> a : {x.P(x)}";
-by (rtac (mem_Collect_eq RS ssubst) 1);
+by (stac mem_Collect_eq 1);
 by (rtac prem 1);
 qed "CollectI";
 
@@ -350,10 +350,10 @@
 bind_thm ("singletonE", make_elim singletonD);
 
 qed_goal "singleton_iff" thy "(b : {a}) = (b=a)" (fn _ => [
-	rtac iffI 1,
-	etac singletonD 1,
-	hyp_subst_tac 1,
-	rtac singletonI 1]);
+        rtac iffI 1,
+        etac singletonD 1,
+        hyp_subst_tac 1,
+        rtac singletonI 1]);
 
 val [major] = goal Set.thy "{a}={b} ==> a=b";
 by (rtac (major RS equalityD1 RS subsetD RS singletonD) 1);
@@ -502,7 +502,7 @@
 
 
 val mem_simps = [insert_iff, empty_iff, Un_iff, Int_iff, Compl_iff, Diff_iff, 
-		 mem_Collect_eq];
+                 mem_Collect_eq];
 
 (*Not for Addsimps -- it can cause goals to blow up!*)
 goal Set.thy "(a : (if Q then x else y)) = ((Q --> a:x) & (~Q --> a : y))";