src/Pure/Tools/update_theorems.scala
changeset 75394 42267c650205
parent 75393 87ebf5a50283
child 75906 2167b9e3157a
--- a/src/Pure/Tools/update_theorems.scala	Fri Apr 01 17:06:10 2022 +0200
+++ b/src/Pure/Tools/update_theorems.scala	Fri Apr 01 23:19:12 2022 +0200
@@ -30,8 +30,9 @@
   /* Isabelle tool wrapper */
 
   val isabelle_tool = Isabelle_Tool("update_theorems", "update toplevel theorem keywords",
-    Scala_Project.here, args => {
-    val getopts = Getopts("""
+    Scala_Project.here,
+    { args =>
+      val getopts = Getopts("""
 Usage: isabelle update_theorems [FILES|DIRS...]
 
   Recursively find .thy files and update toplevel theorem keywords:
@@ -44,12 +45,12 @@
   Old versions of files are preserved by appending "~~".
 """)
 
-    val specs = getopts(args)
-    if (specs.isEmpty) getopts.usage()
+      val specs = getopts(args)
+      if (specs.isEmpty) getopts.usage()
 
-    for {
-      spec <- specs
-      file <- File.find_files(Path.explode(spec).file, file => file.getName.endsWith(".thy"))
-    } update_theorems(File.path(file))
-  })
+      for {
+        spec <- specs
+        file <- File.find_files(Path.explode(spec).file, file => file.getName.endsWith(".thy"))
+      } update_theorems(File.path(file))
+    })
 }