src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 46105 9abb756352a6
parent 46104 eb85282db54e
child 46106 73e2c70980df
equal deleted inserted replaced
46104:eb85282db54e 46105:9abb756352a6
   185 inductive odd where
   185 inductive odd where
   186 "odd 1" |
   186 "odd 1" |
   187 "\<lbrakk>odd m; even n\<rbrakk> \<Longrightarrow> odd (m + n)"
   187 "\<lbrakk>odd m; even n\<rbrakk> \<Longrightarrow> odd (m + n)"
   188 
   188 
   189 lemma "odd n \<Longrightarrow> odd (n - 2)"
   189 lemma "odd n \<Longrightarrow> odd (n - 2)"
   190 nitpick [card nat = 10, show_consts, expect = genuine]
   190 nitpick [card nat = 4, show_consts, expect = genuine]
   191 oops
   191 oops
   192 
   192 
   193 subsection {* 2.9. Coinductive Datatypes *}
   193 subsection {* 2.9. Coinductive Datatypes *}
   194 
   194 
   195 (* Lazy lists are defined in Andreas Lochbihler's "Coinductive" AFP entry. Since
   195 (* Lazy lists are defined in Andreas Lochbihler's "Coinductive" AFP entry. Since