src/HOL/Set.ML
changeset 5490 85855f65d0c6
parent 5450 fe9d103464a4
child 5521 7970832271cc
--- a/src/HOL/Set.ML	Tue Sep 15 13:09:23 1998 +0200
+++ b/src/HOL/Set.ML	Tue Sep 15 15:04:07 1998 +0200
@@ -295,19 +295,19 @@
 
 section "Set complement -- Compl";
 
-qed_goalw "Compl_iff" Set.thy [Compl_def] "(c : Compl(A)) = (c~:A)"
+qed_goalw "Compl_iff" Set.thy [Compl_def] "(c : -A) = (c~:A)"
  (fn _ => [ (Blast_tac 1) ]);
 
 Addsimps [Compl_iff];
 
-val prems = Goalw [Compl_def] "[| c:A ==> False |] ==> c : Compl(A)";
+val prems = Goalw [Compl_def] "[| c:A ==> False |] ==> c : -A";
 by (REPEAT (ares_tac (prems @ [CollectI,notI]) 1));
 qed "ComplI";
 
 (*This form, with negated conclusion, works well with the Classical prover.
   Negated assumptions behave like formulae on the right side of the notional
   turnstile...*)
-Goalw [Compl_def] "c : Compl(A) ==> c~:A";
+Goalw [Compl_def] "c : -A ==> c~:A";
 by (etac CollectD 1);
 qed "ComplD";