| author | haftmann | 
| Thu, 16 Nov 2017 11:30:23 +0100 | |
| changeset 67078 | 6a85b8a9c28c | 
| parent 60500 | 903bb1495239 | 
| child 69593 | 3dda49e08b9d | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Library/Code_Prolog.thy Author: Lukas Bulwahn, TUM 2010 *) section \<open>Code generation of prolog programs\<close> theory Code_Prolog imports Main keywords "values_prolog" :: diag begin ML_file "~~/src/HOL/Tools/Predicate_Compile/code_prolog.ML" section \<open>Setup for Numerals\<close> setup \<open>Predicate_Compile_Data.ignore_consts [@{const_name numeral}]\<close> setup \<open>Predicate_Compile_Data.keep_functions [@{const_name numeral}]\<close> end