# HG changeset patch # User blanchet # Date 1280849394 -7200 # Node ID 6a221fffbc8a7dcf5f83a1010b1ff32d0d5be85e # Parent e3bb14be0931198c567f9717577771af97fa2305 minor changes diff -r e3bb14be0931 -r 6a221fffbc8a src/HOL/Nitpick_Examples/Manual_Nits.thy --- a/src/HOL/Nitpick_Examples/Manual_Nits.thy Tue Aug 03 17:29:27 2010 +0200 +++ b/src/HOL/Nitpick_Examples/Manual_Nits.thy Tue Aug 03 17:29:54 2010 +0200 @@ -158,7 +158,7 @@ oops lemma "\n \ 49. even n \ even (Suc n)" -nitpick [card nat = 50, unary_ints, verbose, expect = genuine] +nitpick [card nat = 50, unary_ints, expect = genuine] oops inductive even' where @@ -192,8 +192,9 @@ subsection {* 3.9. Coinductive Datatypes *} (* Lazy lists are defined in Andreas Lochbihler's "Coinductive" AFP entry. Since -we cannot rely on its presence, we expediently provide our own axiomatization. -The examples also work unchanged with Lochbihler's "Coinductive_List" theory. *) + we cannot rely on its presence, we expediently provide our own + axiomatization. The examples also work unchanged with Lochbihler's + "Coinductive_List" theory. *) typedef 'a llist = "UNIV\('a list + (nat \ 'a)) set" by auto @@ -225,7 +226,7 @@ lemma "\xs = LCons a xs; ys = LCons a ys\ \ xs = ys" nitpick [bisim_depth = -1, show_datatypes, expect = quasi_genuine] -nitpick [expect = none] +nitpick [card = 1\5, expect = none] sorry subsection {* 3.10. Boxing *} @@ -268,7 +269,6 @@ lemma "length xs = length ys \ rev (zip xs ys) = zip xs (rev ys)" nitpick [verbose, expect = genuine] -nitpick [card = 8, verbose, expect = genuine] oops lemma "\g. \x\'b. g (f x) = x \ \y\'a. \x. y = f x" @@ -284,19 +284,19 @@ "n \ reach \ n + 2 \ reach" lemma "n \ reach \ 2 dvd n" -nitpick [card = 1\5, bits = 1\5, expect = none] +(* nitpick *) apply (induct set: reach) apply auto - nitpick [card = 1\5, bits = 1\5, expect = none] + nitpick [card = 1\4, bits = 1\4, expect = none] apply (thin_tac "n \ reach") nitpick [expect = genuine] oops lemma "n \ reach \ 2 dvd n \ n \ 0" -nitpick [card = 1\5, bits = 1\5, expect = none] +(* nitpick *) apply (induct set: reach) apply auto - nitpick [card = 1\5, bits = 1\5, expect = none] + nitpick [card = 1\4, bits = 1\4, expect = none] apply (thin_tac "n \ reach") nitpick [expect = genuine] oops @@ -335,7 +335,7 @@ case Leaf thus ?case by simp next case (Branch t u) thus ?case - nitpick [non_std, card = 1\5, expect = none] + nitpick [non_std, card = 1\4, expect = none] by auto qed