src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 67414 c46b3f9f79ea
parent 67399 eab6ce8368fa
child 68249 949d93804740
equal deleted inserted replaced
67413:2555713586c8 67414:c46b3f9f79ea
   440 sorry
   440 sorry
   441 
   441 
   442 primrec insort\<^sub>1 where
   442 primrec insort\<^sub>1 where
   443 "insort\<^sub>1 \<Lambda> x = N x 1 \<Lambda> \<Lambda>" |
   443 "insort\<^sub>1 \<Lambda> x = N x 1 \<Lambda> \<Lambda>" |
   444 "insort\<^sub>1 (N y k t u) x =
   444 "insort\<^sub>1 (N y k t u) x =
   445  (* (split \<circ> skew) *) (N y k (if x < y then insort\<^sub>1 t x else t)
   445  \<^cancel>\<open>(split \<circ> skew)\<close> (N y k (if x < y then insort\<^sub>1 t x else t)
   446                              (if x > y then insort\<^sub>1 u x else u))"
   446                              (if x > y then insort\<^sub>1 u x else u))"
   447 
   447 
   448 theorem wf_insort\<^sub>1: "wf t \<Longrightarrow> wf (insort\<^sub>1 t x)"
   448 theorem wf_insort\<^sub>1: "wf t \<Longrightarrow> wf (insort\<^sub>1 t x)"
   449 nitpick [expect = genuine]
   449 nitpick [expect = genuine]
   450 oops
   450 oops