src/HOL/Library/Refute.thy
changeset 63432 ba7901e94e7b
parent 60500 903bb1495239
child 69605 a96320074298
--- a/src/HOL/Library/Refute.thy	Mon Jul 11 09:45:10 2016 +0200
+++ b/src/HOL/Library/Refute.thy	Mon Jul 11 09:57:20 2016 +0200
@@ -9,7 +9,9 @@
 
 theory Refute
 imports Main
-keywords "refute" :: diag and "refute_params" :: thy_decl
+keywords
+  "refute" :: diag and
+  "refute_params" :: thy_decl
 begin
 
 ML_file "refute.ML"