diff -r 54a3db2ed201 -r 903bb1495239 src/HOL/Library/Code_Prolog.thy --- a/src/HOL/Library/Code_Prolog.thy Wed Jun 17 10:57:11 2015 +0200 +++ b/src/HOL/Library/Code_Prolog.thy Wed Jun 17 11:03:05 2015 +0200 @@ -2,7 +2,7 @@ Author: Lukas Bulwahn, TUM 2010 *) -section {* Code generation of prolog programs *} +section \Code generation of prolog programs\ theory Code_Prolog imports Main @@ -11,10 +11,10 @@ ML_file "~~/src/HOL/Tools/Predicate_Compile/code_prolog.ML" -section {* Setup for Numerals *} +section \Setup for Numerals\ -setup {* Predicate_Compile_Data.ignore_consts [@{const_name numeral}] *} +setup \Predicate_Compile_Data.ignore_consts [@{const_name numeral}]\ -setup {* Predicate_Compile_Data.keep_functions [@{const_name numeral}] *} +setup \Predicate_Compile_Data.keep_functions [@{const_name numeral}]\ end