| 61337 |      1 | /*  Title:      Pure/Tools/update_theorems.scala
 | 
|  |      2 |     Author:     Makarius
 | 
|  |      3 | 
 | 
|  |      4 | Update toplevel theorem keywords.
 | 
|  |      5 | */
 | 
|  |      6 | 
 | 
|  |      7 | package isabelle
 | 
|  |      8 | 
 | 
|  |      9 | 
 | 
|  |     10 | object Update_Theorems
 | 
|  |     11 | {
 | 
|  |     12 |   def update_theorems(path: Path)
 | 
|  |     13 |   {
 | 
|  |     14 |     val text0 = File.read(path)
 | 
|  |     15 |     val text1 =
 | 
|  |     16 |       (for (tok <- Token.explode(Keyword.Keywords.empty, text0).iterator)
 | 
|  |     17 |         yield {
 | 
|  |     18 |           tok.source match {
 | 
|  |     19 |             case "theorems" => "lemmas"
 | 
|  |     20 |             case "schematic_theorem" | "schematic_lemma" | "schematic_corollary" =>
 | 
|  |     21 |               "schematic_goal"
 | 
|  |     22 |             case s => s
 | 
|  |     23 |         } }).mkString
 | 
|  |     24 | 
 | 
|  |     25 |     if (text0 != text1) {
 | 
|  |     26 |       Output.writeln("changing " + path)
 | 
|  |     27 |       File.write_backup2(path, text1)
 | 
|  |     28 |     }
 | 
|  |     29 |   }
 | 
|  |     30 | 
 | 
|  |     31 | 
 | 
| 62836 |     32 |   /* Isabelle tool wrapper */
 | 
| 61337 |     33 | 
 | 
| 72763 |     34 |   val isabelle_tool = Isabelle_Tool("update_theorems", "update toplevel theorem keywords",
 | 
|  |     35 |     Scala_Project.here, args =>
 | 
| 61337 |     36 |   {
 | 
| 62836 |     37 |     val getopts = Getopts("""
 | 
| 62450 |     38 | Usage: isabelle update_theorems [FILES|DIRS...]
 | 
|  |     39 | 
 | 
|  |     40 |   Recursively find .thy files and update toplevel theorem keywords:
 | 
|  |     41 | 
 | 
|  |     42 |     theorems             ~>  lemmas
 | 
|  |     43 |     schematic_theorem    ~>  schematic_goal
 | 
|  |     44 |     schematic_lemma      ~>  schematic_goal
 | 
|  |     45 |     schematic_corollary  ~>  schematic_goal
 | 
|  |     46 | 
 | 
|  |     47 |   Old versions of files are preserved by appending "~~".
 | 
|  |     48 | """)
 | 
|  |     49 | 
 | 
| 62836 |     50 |     val specs = getopts(args)
 | 
|  |     51 |     if (specs.isEmpty) getopts.usage()
 | 
| 62450 |     52 | 
 | 
| 62836 |     53 |     for {
 | 
|  |     54 |       spec <- specs
 | 
|  |     55 |       file <- File.find_files(Path.explode(spec).file, file => file.getName.endsWith(".thy"))
 | 
| 68994 |     56 |     } update_theorems(File.path(file))
 | 
| 62836 |     57 |   })
 | 
| 61337 |     58 | }
 |