author | blanchet |
Mon, 21 May 2012 10:39:31 +0200 | |
changeset 47944 | e6b51fab96f7 |
parent 47108 | 2a1953f0d20d |
child 48891 | c0eafbd55de3 |
permissions | -rw-r--r-- |
(* Title: HOL/Library/Code_Prolog.thy Author: Lukas Bulwahn, TUM 2010 *) header {* Code generation of prolog programs *} theory Code_Prolog imports Main uses "~~/src/HOL/Tools/Predicate_Compile/code_prolog.ML" begin section {* Setup for Numerals *} setup {* Predicate_Compile_Data.ignore_consts [@{const_name numeral}, @{const_name neg_numeral}] *} setup {* Predicate_Compile_Data.keep_functions [@{const_name numeral}, @{const_name neg_numeral}] *} end