doc-src/Codegen/Thy/Program.thy
changeset 36176 3fe7e97ccca8
parent 34155 14aaccb399b3
child 36259 9f9b9b14cc7a
equal deleted inserted replaced
36175:5cec4ca719d1 36176:3fe7e97ccca8
   428   likely to be used in such situations.
   428   likely to be used in such situations.
   429 *}
   429 *}
   430 
   430 
   431 subsection {* Inductive Predicates *}
   431 subsection {* Inductive Predicates *}
   432 (*<*)
   432 (*<*)
   433 hide const append
   433 hide_const append
   434 
   434 
   435 inductive append
   435 inductive append
   436 where
   436 where
   437   "append [] ys ys"
   437   "append [] ys ys"
   438 | "append xs ys zs ==> append (x # xs) ys (x # zs)"
   438 | "append xs ys zs ==> append (x # xs) ys (x # zs)"