src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy
author bulwahn
Thu, 29 Jul 2010 17:27:58 +0200
changeset 38080 8c20eb9a388d
parent 38075 3d5e2b7d1374
child 38116 823b1e8bc090
permissions -rw-r--r--
cleaning example file; more natural ordering of variable names

theory Code_Prolog_Examples
imports Predicate_Compile_Alternative_Defs
uses "~~/src/HOL/Tools/Predicate_Compile/code_prolog.ML"
begin

section {* Example append *}

inductive append
where
  "append [] ys ys"
| "append xs ys zs ==> append (x # xs) ys (x # zs)"

code_pred append .

values 3 "{((x::'b list), y, z). append x y z}"

end