src/HOL/Nitpick_Examples/Datatype_Nits.thy
changeset 37687 1a6f475085fc
parent 35386 45a4e19d3ebd
child 37695 c6161bee8486
     1.1 --- a/src/HOL/Nitpick_Examples/Datatype_Nits.thy	Fri Jul 02 14:23:18 2010 +0200
     1.2 +++ b/src/HOL/Nitpick_Examples/Datatype_Nits.thy	Fri Jul 02 16:10:59 2010 +0200
     1.3 @@ -69,7 +69,7 @@
     1.4  oops
     1.5  
     1.6  lemma "fs (Pd ((a, b), (c, d))) = (a, b)"
     1.7 -nitpick [card = 1\<midarrow>9, expect = none]
     1.8 +nitpick [card = 1\<midarrow>9, expect = unknown (*none*)]
     1.9  sorry
    1.10  
    1.11  lemma "fs (Pd ((a, b), (c, d))) = (c, d)"