src/HOL/Library/Code_Prolog.thy
changeset 47108 2a1953f0d20d
parent 38731 2c8a595af43e
child 48891 c0eafbd55de3
--- a/src/HOL/Library/Code_Prolog.thy	Sat Mar 24 16:27:04 2012 +0100
+++ b/src/HOL/Library/Code_Prolog.thy	Sun Mar 25 20:15:39 2012 +0200
@@ -11,8 +11,10 @@
 
 section {* Setup for Numerals *}
 
-setup {* Predicate_Compile_Data.ignore_consts [@{const_name number_of}] *}
-setup {* Predicate_Compile_Data.keep_functions [@{const_name number_of}] *}
+setup {* Predicate_Compile_Data.ignore_consts
+  [@{const_name numeral}, @{const_name neg_numeral}] *}
+
+setup {* Predicate_Compile_Data.keep_functions
+  [@{const_name numeral}, @{const_name neg_numeral}] *}
 
 end
-