added "no_atp" for fact that confuses the SMT normalizer and that doesn't help ATPs anyway
authorblanchet
Thu, 25 Nov 2010 00:17:16 +0100
changeset 40690 3f472e57446a
parent 40689 3a10ce7cd436
child 40691 a68f64f99832
added "no_atp" for fact that confuses the SMT normalizer and that doesn't help ATPs anyway
src/HOL/Nat_Numeral.thy
--- a/src/HOL/Nat_Numeral.thy	Wed Nov 24 23:17:24 2010 +0100
+++ b/src/HOL/Nat_Numeral.thy	Thu Nov 25 00:17:16 2010 +0100
@@ -674,7 +674,7 @@
 lemma nat_number_of_Pls: "Numeral0 = (0::nat)"
   by (simp add: nat_number_of_def)
 
-lemma nat_number_of_Min: "number_of Int.Min = (0::nat)"
+lemma nat_number_of_Min [no_atp]: "number_of Int.Min = (0::nat)"
   apply (simp only: number_of_Min nat_number_of_def nat_zminus_int)
   done