src/HOL/Presburger.thy
changeset 20051 859e7129961b
parent 18202 46af82efd311
child 20217 25b068a99d2b
--- a/src/HOL/Presburger.thy	Sat Jul 08 12:54:38 2006 +0200
+++ b/src/HOL/Presburger.thy	Sat Jul 08 12:54:39 2006 +0200
@@ -9,7 +9,7 @@
 header {* Presburger Arithmetic: Cooper's Algorithm *}
 
 theory Presburger
-imports NatSimprocs SetInterval
+imports NatSimprocs
 uses ("cooper_dec.ML") ("cooper_proof.ML") ("qelim.ML") 
 	("reflected_presburger.ML") ("reflected_cooper.ML") ("presburger.ML")
 begin