src/HOL/Presburger.thy
changeset 15013 34264f5e4691
parent 14981 e73f8140af78
child 15131 c69542757a4d
--- a/src/HOL/Presburger.thy	Wed Jun 30 14:04:58 2004 +0200
+++ b/src/HOL/Presburger.thy	Thu Jul 01 12:29:53 2004 +0200
@@ -969,7 +969,7 @@
 theorem number_of1: "(0::int) <= number_of n \<Longrightarrow> (0::int) <= number_of (n BIT b)"
   by simp
 
-theorem number_of2: "(0::int) <= number_of bin.Pls" by simp
+theorem number_of2: "(0::int) <= Numeral0" by simp
 
 theorem Suc_plus1: "Suc n = n + 1" by simp