tuned whitespace;
authorwenzelm
Sat, 28 Nov 2020 23:30:25 +0100
changeset 72766 47ffeb3448f4
parent 72765 f34f5c057c9e
child 72767 f6bf65554764
tuned whitespace;
src/HOL/SPARK/SPARK_Setup.thy
--- a/src/HOL/SPARK/SPARK_Setup.thy	Sat Nov 28 23:28:56 2020 +0100
+++ b/src/HOL/SPARK/SPARK_Setup.thy	Sat Nov 28 23:30:25 2020 +0100
@@ -6,14 +6,12 @@
 *)
 
 theory SPARK_Setup
-  imports
-  "HOL-Library.Word"
-keywords
-  "spark_open_vcg" :: thy_load (spark_vcg) and
-  "spark_open" :: thy_load (spark_siv) and
-  "spark_proof_functions" "spark_types" "spark_end" :: thy_decl and
-  "spark_vc" :: thy_goal and
-  "spark_status" :: diag
+  imports "HOL-Library.Word"
+  keywords "spark_open_vcg" :: thy_load (spark_vcg)
+    and "spark_open" :: thy_load (spark_siv)
+    and "spark_proof_functions" "spark_types" "spark_end" :: thy_decl
+    and "spark_vc" :: thy_goal
+    and "spark_status" :: diag
 begin
 
 ML_file \<open>Tools/fdl_lexer.ML\<close>