fixed import: requires ContNotDenum;
authorwenzelm
Wed, 10 Dec 2008 23:54:03 +0100
changeset 29044 45dfd04a972e
parent 29043 409d1ca929b5
child 29050 cc9a25916582
fixed import: requires ContNotDenum;
src/HOL/Import/HOL4Compat.thy
--- a/src/HOL/Import/HOL4Compat.thy	Wed Dec 10 23:13:21 2008 +0100
+++ b/src/HOL/Import/HOL4Compat.thy	Wed Dec 10 23:54:03 2008 +0100
@@ -3,7 +3,7 @@
     Author:     Sebastian Skalberg (TU Muenchen)
 *)
 
-theory HOL4Compat imports HOL4Setup Divides Primes Real 
+theory HOL4Compat imports HOL4Setup Divides Primes Real ContNotDenum
 begin
 
 lemma EXISTS_UNIQUE_DEF: "(Ex1 P) = (Ex P & (ALL x y. P x & P y --> (x = y)))"