fix proof
authorhuffman
Tue, 06 Sep 2005 20:53:27 +0200
changeset 17292 5c613b64bf0a
parent 17291 94f6113fe9ed
child 17293 ecf182ccc3ca
fix proof
src/HOL/Complex/CStar.thy
--- a/src/HOL/Complex/CStar.thy	Tue Sep 06 19:28:58 2005 +0200
+++ b/src/HOL/Complex/CStar.thy	Tue Sep 06 20:53:27 2005 +0200
@@ -186,6 +186,7 @@
 
 lemma InternalCSets_UNIV_diff:
     "X \<in> InternalCSets ==> UNIV - X \<in> InternalCSets"
+apply (subgoal_tac "UNIV - X = - X")
 by (auto intro: InternalCSets_Compl)
 
 text{*Nonstandard extension of a set (defined using a constant sequence) as a special case of an internal set*}