| author | paulson <lp15@cam.ac.uk> |
| Mon, 17 Mar 2014 15:48:30 +0000 | |
| changeset 56178 | 2a6f58938573 |
| parent 55447 | aa41ecbdc205 |
| child 58881 | b9556a055632 |
| 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 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