| author | wenzelm | 
| Tue, 08 Feb 2011 21:12:27 +0100 | |
| changeset 41734 | d92cc39097e6 | 
| parent 38731 | 2c8a595af43e | 
| child 47108 | 2a1953f0d20d | 
| 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 number_of}] *} setup {* Predicate_Compile_Data.keep_functions [@{const_name number_of}] *} end