| author | noschinl | 
| Fri, 17 Apr 2015 11:12:19 +0200 | |
| changeset 60109 | 22389d4cdd6b | 
| parent 58881 | b9556a055632 | 
| child 60500 | 903bb1495239 | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Library/Code_Prolog.thy Author: Lukas Bulwahn, TUM 2010 *) section {* Code generation of prolog programs *} theory Code_Prolog imports Main keywords "values_prolog" :: diag begin ML_file "~~/src/HOL/Tools/Predicate_Compile/code_prolog.ML" section {* Setup for Numerals *} setup {* Predicate_Compile_Data.ignore_consts [@{const_name numeral}] *} setup {* Predicate_Compile_Data.keep_functions [@{const_name numeral}] *} end