src/HOL/Nitpick_Examples/Typedef_Nits.thy
changeset 39362 ee65900bfced
parent 38542 c9599ce8cbfc
child 40341 03156257040f
--- a/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Tue Sep 14 14:12:18 2010 +0200
+++ b/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Tue Sep 14 14:22:49 2010 +0200
@@ -64,7 +64,7 @@
 oops
 
 lemma "x \<noteq> (y\<Colon>bool bounded) \<Longrightarrow> z = x \<or> z = y"
-nitpick [expect = none]
+nitpick [expect = potential] (* unfortunate *)
 sorry
 
 lemma "x \<noteq> (y\<Colon>(bool \<times> bool) bounded) \<Longrightarrow> z = x \<or> z = y"
@@ -162,10 +162,6 @@
 nitpick [card = 1, unary_ints, max_potential = 0, expect = none]
 by (rule Zero_int_def_raw)
 
-lemma "Abs_Integ (Rep_Integ a) = a"
-nitpick [card = 1, unary_ints, max_potential = 0, expect = none]
-by (rule Rep_Integ_inverse)
-
 lemma "Abs_list (Rep_list a) = a"
 nitpick [card = 1\<midarrow>2, expect = none]
 by (rule Rep_list_inverse)