src/HOL/Predicate_Compile.thy
changeset 63432 ba7901e94e7b
parent 62390 842917225d56
child 67613 ce654b0e6d69
--- a/src/HOL/Predicate_Compile.thy	Mon Jul 11 09:45:10 2016 +0200
+++ b/src/HOL/Predicate_Compile.thy	Mon Jul 11 09:57:20 2016 +0200
@@ -6,7 +6,9 @@
 
 theory Predicate_Compile
 imports Random_Sequence Quickcheck_Exhaustive
-keywords "code_pred" :: thy_goal and "values" :: diag
+keywords
+  "code_pred" :: thy_goal and
+  "values" :: diag
 begin
 
 ML_file "Tools/Predicate_Compile/predicate_compile_aux.ML"