--- a/src/HOL/Tools/Predicate_Compile/code_prolog.ML Sun Mar 13 14:51:38 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/code_prolog.ML Sun Mar 13 15:10:00 2011 +0100
@@ -1,7 +1,8 @@
(* Title: HOL/Tools/Predicate_Compile/code_prolog.ML
Author: Lukas Bulwahn, TU Muenchen
-Prototype of an code generator for logic programming languages (a.k.a. Prolog)
+Prototype of an code generator for logic programming languages
+(a.k.a. Prolog).
*)
signature CODE_PROLOG =
--- a/src/HOL/Tools/Predicate_Compile/core_data.ML Sun Mar 13 14:51:38 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/core_data.ML Sun Mar 13 15:10:00 2011 +0100
@@ -1,9 +1,9 @@
(* Title: HOL/Tools/Predicate_Compile/core_data.ML
Author: Lukas Bulwahn, TU Muenchen
-Data of the predicate compiler core
+Data of the predicate compiler core.
+*)
-*)
signature CORE_DATA =
sig
type mode = Predicate_Compile_Aux.mode
--- a/src/HOL/Tools/Predicate_Compile/mode_inference.ML Sun Mar 13 14:51:38 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/mode_inference.ML Sun Mar 13 15:10:00 2011 +0100
@@ -1,8 +1,7 @@
(* Title: HOL/Tools/Predicate_Compile/mode_inference.ML
Author: Lukas Bulwahn, TU Muenchen
-Mode inference for the predicate compiler
-
+Mode inference for the predicate compiler.
*)
signature MODE_INFERENCE =
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile.ML Sun Mar 13 14:51:38 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile.ML Sun Mar 13 15:10:00 2011 +0100
@@ -1,7 +1,8 @@
(* Title: HOL/Tools/Predicate_Compile/predicate_compile.ML
Author: Lukas Bulwahn, TU Muenchen
-Entry point for the predicate compiler; definition of Toplevel commands code_pred and values
+Entry point for the predicate compiler; definition of Toplevel
+commands code_pred and values.
*)
signature PREDICATE_COMPILE =
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_compilations.ML Sun Mar 13 14:51:38 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_compilations.ML Sun Mar 13 15:10:00 2011 +0100
@@ -1,7 +1,7 @@
(* Title: HOL/Tools/Predicate_Compile/predicate_compile_compilations.ML
Author: Lukas Bulwahn, TU Muenchen
-Structures for different compilations of the predicate compiler
+Structures for different compilations of the predicate compiler.
*)
structure PredicateCompFuns =