src/HOL/Presburger.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 16417 9bc16273c2d4
--- a/src/HOL/Presburger.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Presburger.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -9,7 +9,7 @@
 header {* Presburger Arithmetic: Cooper's Algorithm *}
 
 theory Presburger
-import NatSimprocs SetInterval
+imports NatSimprocs SetInterval
 files ("cooper_dec.ML") ("cooper_proof.ML") ("qelim.ML") ("presburger.ML")
 begin