src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 45970 b6d0cff57d96
parent 45694 4a8743618257
child 46104 eb85282db54e
equal deleted inserted replaced
45969:562e99c3d316 45970:b6d0cff57d96
   177 oops
   177 oops
   178 
   178 
   179 coinductive nats where
   179 coinductive nats where
   180 "nats (x\<Colon>nat) \<Longrightarrow> nats x"
   180 "nats (x\<Colon>nat) \<Longrightarrow> nats x"
   181 
   181 
   182 lemma "nats = {0, 1, 2, 3, 4}"
   182 lemma "nats = (\<lambda>n. n \<in> {0, 1, 2, 3, 4})"
   183 nitpick [card nat = 10, show_consts, expect = genuine]
   183 nitpick [card nat = 10, show_consts, expect = genuine]
   184 oops
   184 oops
   185 
   185 
   186 inductive odd where
   186 inductive odd where
   187 "odd 1" |
   187 "odd 1" |