src/HOL/Tools/Qelim/cooper.ML
changeset 36701 787c33a0e468
parent 36527 68a837d1a754
child 36717 2a72455be88b
--- a/src/HOL/Tools/Qelim/cooper.ML	Thu May 06 16:32:20 2010 +0200
+++ b/src/HOL/Tools/Qelim/cooper.ML	Thu May 06 16:32:21 2010 +0200
@@ -3,7 +3,7 @@
 *)
 
 signature COOPER =
- sig
+sig
   val cooper_conv : Proof.context -> conv
   exception COOPER of string * exn
 end;
@@ -12,7 +12,6 @@
 struct
 
 open Conv;
-open Normalizer;
 
 exception COOPER of string * exn;
 fun simp_thms_conv ctxt =