src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 37477 e482320bcbfe
parent 36268 65aabc2c89ae
child 38184 6a221fffbc8a
--- a/src/HOL/Nitpick_Examples/Manual_Nits.thy	Mon Jun 21 11:15:21 2010 +0200
+++ b/src/HOL/Nitpick_Examples/Manual_Nits.thy	Mon Jun 21 11:16:00 2010 +0200
@@ -7,13 +7,17 @@
 
 header {* Examples from the Nitpick Manual *}
 
+(* The "expect" arguments to Nitpick in this theory and the other example
+   theories are there so that the example can also serve as a regression test
+   suite. *)
+
 theory Manual_Nits
 imports Main Quotient_Product RealDef
 begin
 
 chapter {* 3. First Steps *}
 
-nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1]
+nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60 s]
 
 subsection {* 3.1. Propositional Logic *}
 
@@ -379,7 +383,7 @@
 
 theorem S\<^isub>3_sound:
 "w \<in> S\<^isub>3 \<longrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
-nitpick [card = 1\<midarrow>6, expect = none]
+nitpick [card = 1\<midarrow>5, expect = none]
 sorry
 
 theorem S\<^isub>3_complete:
@@ -398,19 +402,19 @@
 
 theorem S\<^isub>4_sound:
 "w \<in> S\<^isub>4 \<longrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
-nitpick [card = 1\<midarrow>6, expect = none]
+nitpick [card = 1\<midarrow>5, expect = none]
 sorry
 
 theorem S\<^isub>4_complete:
 "length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] \<longrightarrow> w \<in> S\<^isub>4"
-nitpick [card = 1\<midarrow>6, expect = none]
+nitpick [card = 1\<midarrow>5, expect = none]
 sorry
 
 theorem S\<^isub>4_A\<^isub>4_B\<^isub>4_sound_and_complete:
 "w \<in> S\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b]"
 "w \<in> A\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = a] = length [x \<leftarrow> w. x = b] + 1"
 "w \<in> B\<^isub>4 \<longleftrightarrow> length [x \<leftarrow> w. x = b] = length [x \<leftarrow> w. x = a] + 1"
-nitpick [card = 1\<midarrow>6, expect = none]
+nitpick [card = 1\<midarrow>5, expect = none]
 sorry
 
 subsection {* 4.2. AA Trees *}