diff -r eef345eff987 -r 69e55066dbca src/HOL/Presburger.thy --- a/src/HOL/Presburger.thy Thu May 31 18:16:51 2007 +0200 +++ b/src/HOL/Presburger.thy Thu May 31 18:16:52 2007 +0200 @@ -9,7 +9,7 @@ header {* Presburger Arithmetic: Cooper's Algorithm *} theory Presburger -imports "Integ/NatSimprocs" SetInterval +imports NatSimprocs SetInterval uses ("Tools/Presburger/cooper_dec.ML") ("Tools/Presburger/cooper_proof.ML")