diff -r 11fca474d87a -r b1278ed3cd46 src/HOL/ex/PresburgerEx.thy --- a/src/HOL/ex/PresburgerEx.thy Sat Nov 04 18:57:49 2017 +0100 +++ b/src/HOL/ex/PresburgerEx.thy Sat Nov 04 19:17:19 2017 +0100 @@ -5,7 +5,7 @@ section \Some examples for Presburger Arithmetic\ theory PresburgerEx -imports HOL.Presburger +imports Main begin lemma "\m n ja ia. \\ m \ j; \ (n::nat) \ i; (e::nat) \ 0; Suc j \ ja\ \ \m. \ja ia. m \ ja \ (if j = ja \ i = ia then e else 0) = 0" by presburger