src/HOL/Nitpick_Examples/Integer_Nits.thy
changeset 47108 2a1953f0d20d
parent 46090 f1796596ef60
child 47109 db5026631799
--- a/src/HOL/Nitpick_Examples/Integer_Nits.thy	Sat Mar 24 16:27:04 2012 +0100
+++ b/src/HOL/Nitpick_Examples/Integer_Nits.thy	Sun Mar 25 20:15:39 2012 +0200
@@ -198,7 +198,18 @@
 lemma "-5 * 55 > (-260::int)"
 nitpick [unary_ints, expect = none]
 nitpick [binary_ints, expect = none]
+(* BROKEN
+Nitpicking formula...
+Trying 5 scopes:
+  card bin = 1, card int = 1, and bits = 9;
+  card bin = 2, card int = 2, and bits = 9;
+  card bin = 3, card int = 3, and bits = 9;
+  card bin = 4, card int = 4, and bits = 9;
+  card bin = 5, card int = 5, and bits = 9.
+Nitpick found no counterexample.
+*** Unexpected outcome: "none".
 nitpick [binary_ints, bits = 9, expect = genuine]
+*)
 oops
 
 lemma "nat (of_nat n) = n"