author | hoelzl |
Thu, 17 Jan 2013 11:59:12 +0100 | |
changeset 50936 | b28f258ebc1a |
parent 48891 | c0eafbd55de3 |
child 54489 | 03ff4d1e6784 |
permissions | -rw-r--r-- |
38117 | 1 |
(* Title: HOL/Library/Code_Prolog.thy |
2 |
Author: Lukas Bulwahn, TUM 2010 |
|
3 |
*) |
|
4 |
||
5 |
header {* Code generation of prolog programs *} |
|
6 |
||
7 |
theory Code_Prolog |
|
8 |
imports Main |
|
9 |
begin |
|
10 |
||
48891 | 11 |
ML_file "~~/src/HOL/Tools/Predicate_Compile/code_prolog.ML" |
12 |
||
38731
2c8a595af43e
invocation of values for prolog execution does not require invocation of code_pred anymore
bulwahn
parents:
38117
diff
changeset
|
13 |
section {* Setup for Numerals *} |
2c8a595af43e
invocation of values for prolog execution does not require invocation of code_pred anymore
bulwahn
parents:
38117
diff
changeset
|
14 |
|
47108
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
huffman
parents:
38731
diff
changeset
|
15 |
setup {* Predicate_Compile_Data.ignore_consts |
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
huffman
parents:
38731
diff
changeset
|
16 |
[@{const_name numeral}, @{const_name neg_numeral}] *} |
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
huffman
parents:
38731
diff
changeset
|
17 |
|
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
huffman
parents:
38731
diff
changeset
|
18 |
setup {* Predicate_Compile_Data.keep_functions |
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
huffman
parents:
38731
diff
changeset
|
19 |
[@{const_name numeral}, @{const_name neg_numeral}] *} |
38731
2c8a595af43e
invocation of values for prolog execution does not require invocation of code_pred anymore
bulwahn
parents:
38117
diff
changeset
|
20 |
|
38117 | 21 |
end |