Quot/Examples/IntEx.thy
changeset 656 c86a47d4966e
parent 652 d8f07b5bcfae
child 663 0dd10a900cae
equal deleted inserted replaced
655:5ededdde9e9f 656:c86a47d4966e
   319 apply simp
   319 apply simp
   320 done
   320 done
   321 
   321 
   322 lemma "map (\<lambda>x. PLUS x ZERO) l = l"
   322 lemma "map (\<lambda>x. PLUS x ZERO) l = l"
   323 apply(lifting lam_tst4)
   323 apply(lifting lam_tst4)
   324 apply(cleaning)
   324 done
   325 sorry
       
   326 
   325 
   327 end
   326 end