src/HOL/Nitpick_Examples/Typedef_Nits.thy
changeset 35386 45a4e19d3ebd
parent 35312 99cd1f96b400
child 35387 4356263e0bdd
--- a/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Thu Feb 25 16:33:39 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Fri Feb 26 16:49:46 2010 +0100
@@ -64,7 +64,7 @@
 oops
 
 lemma "x \<noteq> (y\<Colon>bool bounded) \<Longrightarrow> z = x \<or> z = y"
-nitpick [expect = none]
+nitpick [fast_descrs (* ### FIXME *), expect = none]
 sorry
 
 lemma "x \<noteq> (y\<Colon>(bool \<times> bool) bounded) \<Longrightarrow> z = x \<or> z = y"