src/HOL/ex/PresburgerEx.thy
changeset 16417 9bc16273c2d4
parent 15075 a6cd1a454751
child 17388 495c799df31d
--- a/src/HOL/ex/PresburgerEx.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/ex/PresburgerEx.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 Some examples for Presburger Arithmetic
 *)
 
-theory PresburgerEx = Main:
+theory PresburgerEx imports Main begin
 
 theorem "(\<forall>(y::int). 3 dvd y) ==> \<forall>(x::int). b < x --> a \<le> x"
   by presburger