author | wenzelm |
Sat, 01 Jul 2023 16:42:57 +0200 | |
changeset 78237 | c2c59de57df9 |
parent 78233 | 1a12e6246212 |
child 78280 | 865b44cbaad1 |
permissions | -rw-r--r-- |
50686 | 1 |
/* Title: Pure/Tools/build.scala |
48276 | 2 |
Author: Makarius |
57923 | 3 |
Options: :folding=explicit: |
48276 | 4 |
|
77553 | 5 |
Command-line tools to build and manage Isabelle sessions. |
48276 | 6 |
*/ |
7 |
||
8 |
package isabelle |
|
9 |
||
77553 | 10 |
import scala.collection.mutable |
11 |
import scala.util.matching.Regex |
|
12 |
||
48276 | 13 |
|
75393 | 14 |
object Build { |
77553 | 15 |
/** "isabelle build" **/ |
16 |
||
78232 | 17 |
/* options */ |
18 |
||
19 |
def hostname(options: Options): String = |
|
20 |
Isabelle_System.hostname(options.string("build_hostname")) |
|
21 |
||
22 |
def engine_name(options: Options): String = options.string("build_engine") |
|
23 |
||
24 |
||
25 |
||
77330
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
26 |
/* results */ |
48424 | 27 |
|
77311 | 28 |
object Results { |
29 |
def apply(context: Build_Process.Context, results: Map[String, Process_Result]): Results = |
|
77453 | 30 |
new Results(context.store, context.build_deps, results) |
77311 | 31 |
} |
32 |
||
33 |
class Results private( |
|
78178 | 34 |
val store: Store, |
76209 | 35 |
val deps: Sessions.Deps, |
77253
792dad9cb04f
clarified data structure: absorb Option[Process_Result] into Process_Result, e.g. to simplify database storage;
wenzelm
parents:
77252
diff
changeset
|
36 |
results: Map[String, Process_Result] |
76198
fb4215da4919
clarified presentation_sessions: work with partial results;
wenzelm
parents:
76197
diff
changeset
|
37 |
) { |
76206
769a7cd5a16a
clarified signature: re-use store/cache from build results;
wenzelm
parents:
76202
diff
changeset
|
38 |
def cache: Term.Cache = store.cache |
769a7cd5a16a
clarified signature: re-use store/cache from build results;
wenzelm
parents:
76202
diff
changeset
|
39 |
|
77311 | 40 |
def sessions_ok: List[String] = |
41 |
(for { |
|
42 |
name <- deps.sessions_structure.build_topological_order.iterator |
|
43 |
result <- results.get(name) if result.ok |
|
44 |
} yield name).toList |
|
45 |
||
77250
22016642d6af
clarified data structure: use static info from deps, not dynamic results;
wenzelm
parents:
77246
diff
changeset
|
46 |
def info(name: String): Sessions.Info = deps.sessions_structure(name) |
62403 | 47 |
def sessions: Set[String] = results.keySet |
77253
792dad9cb04f
clarified data structure: absorb Option[Process_Result] into Process_Result, e.g. to simplify database storage;
wenzelm
parents:
77252
diff
changeset
|
48 |
def cancelled(name: String): Boolean = !results(name).defined |
792dad9cb04f
clarified data structure: absorb Option[Process_Result] into Process_Result, e.g. to simplify database storage;
wenzelm
parents:
77252
diff
changeset
|
49 |
def apply(name: String): Process_Result = results(name).strict |
792dad9cb04f
clarified data structure: absorb Option[Process_Result] into Process_Result, e.g. to simplify database storage;
wenzelm
parents:
77252
diff
changeset
|
50 |
val rc: Int = results.valuesIterator.map(_.strict.rc).foldLeft(Process_Result.RC.ok)(_ max _) |
74306 | 51 |
def ok: Boolean = rc == Process_Result.RC.ok |
62406 | 52 |
|
76202 | 53 |
def unfinished: List[String] = sessions.iterator.filterNot(apply(_).ok).toList.sorted |
76199 | 54 |
|
62406 | 55 |
override def toString: String = rc.toString |
62403 | 56 |
} |
57 |
||
77330
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
58 |
|
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
59 |
/* engine */ |
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
60 |
|
78232 | 61 |
object Engine { |
62 |
lazy val services: List[Engine] = |
|
63 |
Isabelle_System.make_services(classOf[Engine]) |
|
64 |
||
65 |
def apply(name: String): Engine = |
|
66 |
services.find(_.name == name).getOrElse(error("Bad build engine " + quote(name))) |
|
67 |
} |
|
68 |
||
77411
149cc77f7348
clafified signature: simplify object-oriented reuse;
wenzelm
parents:
77384
diff
changeset
|
69 |
class Engine(val name: String) extends Isabelle_System.Service { |
77330
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
70 |
override def toString: String = name |
78232 | 71 |
|
72 |
def build_options(options: Options): Options = |
|
73 |
options + "completion_limit=0" + "editor_tracing_messages=0" |
|
74 |
||
75 |
def build_process(build_context: Build_Process.Context, build_progress: Progress): Build_Process = |
|
77505 | 76 |
new Build_Process(build_context, build_progress) |
78232 | 77 |
|
78233 | 78 |
final def build_store(options: Options, cache: Term.Cache = Term.Cache.make()): Store = { |
78232 | 79 |
val store = Store(build_options(options), cache = cache) |
78233 | 80 |
|
81 |
Isabelle_System.make_directory(store.output_dir + Path.basic("log")) |
|
82 |
||
78232 | 83 |
Isabelle_Fonts.init() |
78233 | 84 |
|
78232 | 85 |
store |
86 |
} |
|
87 |
||
88 |
final def run(context: Build_Process.Context, progress: Progress): Results = |
|
89 |
Isabelle_Thread.uninterruptible { |
|
90 |
using(build_process(context, progress)) { build_process => |
|
91 |
Results(context, build_process.run()) |
|
92 |
} |
|
93 |
} |
|
77330
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
94 |
} |
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
95 |
|
77411
149cc77f7348
clafified signature: simplify object-oriented reuse;
wenzelm
parents:
77384
diff
changeset
|
96 |
class Default_Engine extends Engine("") { override def toString: String = "<default>" } |
77330
47eb96592aa2
support alternative build engines, via system option "build_engine";
wenzelm
parents:
77326
diff
changeset
|
97 |
|
77558 | 98 |
|
99 |
/* build */ |
|
100 |
||
62641 | 101 |
def build( |
50404
898cac1dad5e
avoid startup within GUI thread -- it is only required later for dialog;
wenzelm
parents:
50367
diff
changeset
|
102 |
options: Options, |
71981 | 103 |
selection: Sessions.Selection = Sessions.Selection.empty, |
75942
603852abed8f
clarified names: Browser_Info.Config vs. Browser_Info.Context;
wenzelm
parents:
75941
diff
changeset
|
104 |
browser_info: Browser_Info.Config = Browser_Info.Config.none, |
71726
a5fda30edae2
clarified signature: more uniform treatment of stopped/interrupted state;
wenzelm
parents:
71718
diff
changeset
|
105 |
progress: Progress = new Progress, |
65832
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
106 |
check_unknown_files: Boolean = false, |
48511
37999ee01156
remove old output heaps, to ensure that result is valid wrt. check_stamps;
wenzelm
parents:
48509
diff
changeset
|
107 |
build_heap: Boolean = false, |
48595 | 108 |
clean_build: Boolean = false, |
56890 | 109 |
dirs: List[Path] = Nil, |
110 |
select_dirs: List[Path] = Nil, |
|
66968
9991671c98aa
allow to augment session context via explicit session infos;
wenzelm
parents:
66962
diff
changeset
|
111 |
infos: List[Sessions.Info] = Nil, |
64265 | 112 |
numa_shuffling: Boolean = false, |
48509 | 113 |
max_jobs: Int = 1, |
48903 | 114 |
list_files: Boolean = false, |
59891
9ce697050455
added isabelle build option -k, for fast off-line checking of theory sources;
wenzelm
parents:
59811
diff
changeset
|
115 |
check_keywords: Set[String] = Set.empty, |
66841 | 116 |
fresh_build: Boolean = false, |
48509 | 117 |
no_build: Boolean = false, |
66745 | 118 |
soft_build: Boolean = false, |
73805
b73777a0c076
allow build session setup, e.g. for protocol handlers;
wenzelm
parents:
73804
diff
changeset
|
119 |
export_files: Boolean = false, |
76927
da13da82f6f9
treat update_options as part of Sessions.Info meta_digest, for proper re-build of updated sessions;
wenzelm
parents:
76919
diff
changeset
|
120 |
augment_options: String => List[Options.Spec] = _ => Nil, |
77559
4ad322ee6025
clarified signature: support all arguments of Sessions.store();
wenzelm
parents:
77558
diff
changeset
|
121 |
session_setup: (String, Session) => Unit = (_, _) => (), |
4ad322ee6025
clarified signature: support all arguments of Sessions.store();
wenzelm
parents:
77558
diff
changeset
|
122 |
cache: Term.Cache = Term.Cache.make() |
75393 | 123 |
): Results = { |
78232 | 124 |
val build_engine = Engine(engine_name(options)) |
125 |
||
78233 | 126 |
val store = build_engine.build_store(options, cache = cache) |
77557 | 127 |
val build_options = store.options |
69369
6ecc85955e04
prefer "Isabelle DejaVu Sans", even for headless batch-build (session_graph.pdf);
wenzelm
parents:
68957
diff
changeset
|
128 |
|
66745 | 129 |
|
130 |
/* session selection and dependencies */ |
|
65422 | 131 |
|
66961 | 132 |
val full_sessions = |
76927
da13da82f6f9
treat update_options as part of Sessions.Info meta_digest, for proper re-build of updated sessions;
wenzelm
parents:
76919
diff
changeset
|
133 |
Sessions.load_structure(build_options, dirs = dirs, select_dirs = select_dirs, infos = infos, |
da13da82f6f9
treat update_options as part of Sessions.Info meta_digest, for proper re-build of updated sessions;
wenzelm
parents:
76919
diff
changeset
|
134 |
augment_options = augment_options) |
73012
238ddf525da4
clarified HTML presentation, e.g. avoid bulky jobs like HOL or HOL-Analysis in applications;
wenzelm
parents:
72993
diff
changeset
|
135 |
val full_sessions_selection = full_sessions.imports_selection(selection) |
238ddf525da4
clarified HTML presentation, e.g. avoid bulky jobs like HOL or HOL-Analysis in applications;
wenzelm
parents:
72993
diff
changeset
|
136 |
|
75948 | 137 |
val build_deps = { |
66745 | 138 |
val deps0 = |
77521
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
139 |
Sessions.deps(full_sessions.selection(selection), progress = progress, inlined_files = true, |
66962
e1bde71bace6
clarified signature: global_theories is always required;
wenzelm
parents:
66961
diff
changeset
|
140 |
list_files = list_files, check_keywords = check_keywords).check_errors |
66745 | 141 |
|
66841 | 142 |
if (soft_build && !fresh_build) { |
66745 | 143 |
val outdated = |
68204 | 144 |
deps0.sessions_structure.build_topological_order.flatMap(name => |
72634
5cea0993ee4f
clarified access to single database server vs. collection of database files;
wenzelm
parents:
72624
diff
changeset
|
145 |
store.try_open_database(name) match { |
68214 | 146 |
case Some(db) => |
68216 | 147 |
using(db)(store.read_build(_, name)) match { |
77675
9e5f8f6e58a0
more thorough treatment of build prefs, guarded by system option "build_through": avoid accidental rebuild of HOL etc.;
wenzelm
parents:
77674
diff
changeset
|
148 |
case Some(build) if build.ok => |
9e5f8f6e58a0
more thorough treatment of build prefs, guarded by system option "build_through": avoid accidental rebuild of HOL etc.;
wenzelm
parents:
77674
diff
changeset
|
149 |
val session_options = deps0.sessions_structure(name).options |
9e5f8f6e58a0
more thorough treatment of build prefs, guarded by system option "build_through": avoid accidental rebuild of HOL etc.;
wenzelm
parents:
77674
diff
changeset
|
150 |
val session_sources = deps0.sources_shasum(name) |
9e5f8f6e58a0
more thorough treatment of build prefs, guarded by system option "build_through": avoid accidental rebuild of HOL etc.;
wenzelm
parents:
77674
diff
changeset
|
151 |
if (Sessions.eq_sources(session_options, build.sources, session_sources)) None |
9e5f8f6e58a0
more thorough treatment of build prefs, guarded by system option "build_through": avoid accidental rebuild of HOL etc.;
wenzelm
parents:
77674
diff
changeset
|
152 |
else Some(name) |
66745 | 153 |
case _ => Some(name) |
154 |
} |
|
155 |
case None => Some(name) |
|
156 |
}) |
|
68204 | 157 |
|
158 |
Sessions.deps(full_sessions.selection(Sessions.Selection(sessions = outdated)), |
|
70671
cb1776c8e216
clarified signature: retain global session information, unaffected by later restriction;
wenzelm
parents:
70509
diff
changeset
|
159 |
progress = progress, inlined_files = true).check_errors |
66745 | 160 |
} |
68204 | 161 |
else deps0 |
66745 | 162 |
} |
163 |
||
164 |
||
165 |
/* check unknown files */ |
|
48504
21dfd6c04482
actually check source vs. target stamps, based on information from log files;
wenzelm
parents:
48494
diff
changeset
|
166 |
|
65832
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
167 |
if (check_unknown_files) { |
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
168 |
val source_files = |
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
169 |
(for { |
75948 | 170 |
(_, base) <- build_deps.session_bases.iterator |
75741 | 171 |
(path, _) <- base.session_sources.iterator |
65832
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
172 |
} yield path).toList |
76670
b04d45bebbc5
discontinued somewhat pointless dependency: avoid illusion of extra accuracy (see also 09fb749d1a1e and 0f750a6dc754);
wenzelm
parents:
76669
diff
changeset
|
173 |
Mercurial.check_files(source_files)._2 match { |
b04d45bebbc5
discontinued somewhat pointless dependency: avoid illusion of extra accuracy (see also 09fb749d1a1e and 0f750a6dc754);
wenzelm
parents:
76669
diff
changeset
|
174 |
case Nil => |
b04d45bebbc5
discontinued somewhat pointless dependency: avoid illusion of extra accuracy (see also 09fb749d1a1e and 0f750a6dc754);
wenzelm
parents:
76669
diff
changeset
|
175 |
case unknown_files => |
b04d45bebbc5
discontinued somewhat pointless dependency: avoid illusion of extra accuracy (see also 09fb749d1a1e and 0f750a6dc754);
wenzelm
parents:
76669
diff
changeset
|
176 |
progress.echo_warning("Unknown files (not part of the underlying Mercurial repository):" + |
76883 | 177 |
unknown_files.map(File.standard_path).sorted.mkString("\n ", "\n ", "")) |
65832
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
178 |
} |
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
179 |
} |
2fb85623c386
implicitly check for unknown files (not part of a Mercurial repository);
wenzelm
parents:
65831
diff
changeset
|
180 |
|
51220 | 181 |
|
77257 | 182 |
/* build process and results */ |
51220 | 183 |
|
77315
f34559b24277
clarified signature: move all parameters into Build_Process.Context;
wenzelm
parents:
77311
diff
changeset
|
184 |
val build_context = |
78237
c2c59de57df9
clarified static Build_Process.Context vs. dynamic Build_Process.State;
wenzelm
parents:
78233
diff
changeset
|
185 |
Build_Process.Context(store, build_deps, hostname = hostname(build_options), |
c2c59de57df9
clarified static Build_Process.Context vs. dynamic Build_Process.State;
wenzelm
parents:
78233
diff
changeset
|
186 |
build_heap = build_heap, numa_shuffling = numa_shuffling, max_jobs = max_jobs, |
c2c59de57df9
clarified static Build_Process.Context vs. dynamic Build_Process.State;
wenzelm
parents:
78233
diff
changeset
|
187 |
fresh_build = fresh_build, no_build = no_build, session_setup = session_setup, |
c2c59de57df9
clarified static Build_Process.Context vs. dynamic Build_Process.State;
wenzelm
parents:
78233
diff
changeset
|
188 |
master = true) |
77254
8d34f53871b4
clarified signature: make dynamic Queue from static Context;
wenzelm
parents:
77253
diff
changeset
|
189 |
|
48595 | 190 |
if (clean_build) { |
78213
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
191 |
using_optional(store.maybe_open_database_server()) { database_server => |
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
192 |
for (name <- full_sessions.imports_descendants(full_sessions_selection)) { |
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
193 |
store.clean_output(database_server, name) match { |
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
194 |
case None => |
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
195 |
case Some(true) => progress.echo("Cleaned " + name) |
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
196 |
case Some(false) => progress.echo(name + " FAILED to clean") |
fd0430a7b7a4
avoid repeated open_database_server: synchronized transaction_lock;
wenzelm
parents:
78178
diff
changeset
|
197 |
} |
68220
8fc4e3d1df86
clarified store.clean_output: cleanup user_output_dir even in system_mode;
wenzelm
parents:
68219
diff
changeset
|
198 |
} |
48595 | 199 |
} |
200 |
} |
|
201 |
||
78232 | 202 |
val results = build_engine.run(build_context, progress) |
62641 | 203 |
|
69811
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
204 |
if (export_files) { |
76196 | 205 |
for (name <- full_sessions_selection.iterator if results(name).ok) { |
69811
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
206 |
val info = results.info(name) |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
207 |
if (info.export_files.nonEmpty) { |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
208 |
progress.echo("Exporting " + info.name + " ...") |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
209 |
for ((dir, prune, pats) <- info.export_files) { |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
210 |
Export.export_files(store, name, info.dir + dir, |
77521
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
211 |
progress = if (progress.verbose) progress else new Progress, |
69811
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
212 |
export_prune = prune, |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
213 |
export_patterns = pats) |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
214 |
} |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
215 |
} |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
216 |
} |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
217 |
} |
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
218 |
|
76901 | 219 |
val presentation_sessions = |
220 |
results.sessions_ok.filter(name => browser_info.enabled(results.info(name))) |
|
76230 | 221 |
if (presentation_sessions.nonEmpty && !progress.stopped) { |
222 |
Browser_Info.build(browser_info, results.store, results.deps, presentation_sessions, |
|
77521
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
223 |
progress = progress) |
76198
fb4215da4919
clarified presentation_sessions: work with partial results;
wenzelm
parents:
76197
diff
changeset
|
224 |
} |
fb4215da4919
clarified presentation_sessions: work with partial results;
wenzelm
parents:
76197
diff
changeset
|
225 |
|
77521
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
226 |
if (!results.ok && (progress.verbose || !no_build)) { |
76199 | 227 |
progress.echo("Unfinished session(s): " + commas(results.unfinished)) |
62641 | 228 |
} |
229 |
||
230 |
results |
|
48341 | 231 |
} |
232 |
||
233 |
||
77555 | 234 |
/* build logic image */ |
235 |
||
236 |
def build_logic(options: Options, logic: String, |
|
237 |
progress: Progress = new Progress, |
|
238 |
build_heap: Boolean = false, |
|
239 |
dirs: List[Path] = Nil, |
|
240 |
fresh: Boolean = false, |
|
241 |
strict: Boolean = false |
|
242 |
): Int = { |
|
243 |
val selection = Sessions.Selection.session(logic) |
|
244 |
val rc = |
|
245 |
if (!fresh && build(options, selection = selection, |
|
246 |
build_heap = build_heap, no_build = true, dirs = dirs).ok) Process_Result.RC.ok |
|
247 |
else { |
|
248 |
progress.echo("Build started for Isabelle/" + logic + " ...") |
|
249 |
build(options, selection = selection, progress = progress, |
|
250 |
build_heap = build_heap, fresh_build = fresh, dirs = dirs).rc |
|
251 |
} |
|
252 |
if (strict && rc != Process_Result.RC.ok) error("Failed to build Isabelle/" + logic) else rc |
|
253 |
} |
|
254 |
||
255 |
||
77553 | 256 |
/* command-line wrapper */ |
48341 | 257 |
|
77553 | 258 |
val isabelle_tool1 = Isabelle_Tool("build", "build and manage Isabelle sessions", |
75394 | 259 |
Scala_Project.here, |
260 |
{ args => |
|
261 |
var base_sessions: List[String] = Nil |
|
262 |
var select_dirs: List[Path] = Nil |
|
263 |
var numa_shuffling = false |
|
75942
603852abed8f
clarified names: Browser_Info.Config vs. Browser_Info.Context;
wenzelm
parents:
75941
diff
changeset
|
264 |
var browser_info = Browser_Info.Config.none |
75394 | 265 |
var requirements = false |
266 |
var soft_build = false |
|
267 |
var exclude_session_groups: List[String] = Nil |
|
268 |
var all_sessions = false |
|
269 |
var build_heap = false |
|
270 |
var clean_build = false |
|
271 |
var dirs: List[Path] = Nil |
|
272 |
var export_files = false |
|
273 |
var fresh_build = false |
|
274 |
var session_groups: List[String] = Nil |
|
275 |
var max_jobs = 1 |
|
276 |
var check_keywords: Set[String] = Set.empty |
|
277 |
var list_files = false |
|
278 |
var no_build = false |
|
77628 | 279 |
var options = Options.init(specs = Options.Spec.ISABELLE_BUILD_OPTIONS) |
75394 | 280 |
var verbose = false |
281 |
var exclude_sessions: List[String] = Nil |
|
62590 | 282 |
|
75394 | 283 |
val getopts = Getopts(""" |
62590 | 284 |
Usage: isabelle build [OPTIONS] [SESSIONS ...] |
285 |
||
286 |
Options are: |
|
66737
2edc0c42c883
option -B for "isabelle build" and "isabelle imports";
wenzelm
parents:
66736
diff
changeset
|
287 |
-B NAME include session NAME and all descendants |
62590 | 288 |
-D DIR include session directory and select its sessions |
64265 | 289 |
-N cyclic shuffling of NUMA CPU nodes (performance tuning) |
72648 | 290 |
-P DIR enable HTML/PDF presentation in directory (":" for default) |
71807 | 291 |
-R refer to requirements of selected sessions |
66745 | 292 |
-S soft build: only observe changes of sources, not heap images |
62590 | 293 |
-X NAME exclude sessions from group NAME and all descendants |
294 |
-a select all sessions |
|
295 |
-b build heap images |
|
296 |
-c clean build |
|
297 |
-d DIR include session directory |
|
69811
18f61ce86425
clarified 'export_files' in session ROOT: require explicit "isabelle build -e";
wenzelm
parents:
69777
diff
changeset
|
298 |
-e export files from session specification into file-system |
66841 | 299 |
-f fresh build |
62590 | 300 |
-g NAME select session group NAME |
301 |
-j INT maximum number of parallel jobs (default 1) |
|
302 |
-k KEYWORD check theory sources for conflicts with proposed keywords |
|
303 |
-l list session source files |
|
77554
4465d9dff448
clarified terminology of "session build database", while "build database" is the one underlying Build_Process;
wenzelm
parents:
77553
diff
changeset
|
304 |
-n no build -- take existing session build databases |
62590 | 305 |
-o OPTION override Isabelle system OPTION (via NAME=VAL or NAME) |
306 |
-v verbose |
|
307 |
-x NAME exclude session NAME and all descendants |
|
308 |
||
77647 | 309 |
Build and manage Isabelle sessions: ML heaps, session databases, documents. |
62596 | 310 |
|
77647 | 311 |
Notable system options: see "isabelle options -l -t build" |
312 |
||
313 |
Notable system settings: |
|
314 |
""" + Library.indent_lines(4, Build_Log.Settings.show()) + "\n", |
|
75394 | 315 |
"B:" -> (arg => base_sessions = base_sessions ::: List(arg)), |
316 |
"D:" -> (arg => select_dirs = select_dirs ::: List(Path.explode(arg))), |
|
317 |
"N" -> (_ => numa_shuffling = true), |
|
75942
603852abed8f
clarified names: Browser_Info.Config vs. Browser_Info.Context;
wenzelm
parents:
75941
diff
changeset
|
318 |
"P:" -> (arg => browser_info = Browser_Info.Config.make(arg)), |
75394 | 319 |
"R" -> (_ => requirements = true), |
320 |
"S" -> (_ => soft_build = true), |
|
321 |
"X:" -> (arg => exclude_session_groups = exclude_session_groups ::: List(arg)), |
|
322 |
"a" -> (_ => all_sessions = true), |
|
323 |
"b" -> (_ => build_heap = true), |
|
324 |
"c" -> (_ => clean_build = true), |
|
325 |
"d:" -> (arg => dirs = dirs ::: List(Path.explode(arg))), |
|
326 |
"e" -> (_ => export_files = true), |
|
327 |
"f" -> (_ => fresh_build = true), |
|
328 |
"g:" -> (arg => session_groups = session_groups ::: List(arg)), |
|
329 |
"j:" -> (arg => max_jobs = Value.Int.parse(arg)), |
|
330 |
"k:" -> (arg => check_keywords = check_keywords + arg), |
|
331 |
"l" -> (_ => list_files = true), |
|
332 |
"n" -> (_ => no_build = true), |
|
333 |
"o:" -> (arg => options = options + arg), |
|
334 |
"v" -> (_ => verbose = true), |
|
335 |
"x:" -> (arg => exclude_sessions = exclude_sessions ::: List(arg))) |
|
62590 | 336 |
|
75394 | 337 |
val sessions = getopts(args) |
62590 | 338 |
|
75394 | 339 |
val progress = new Console_Progress(verbose = verbose) |
62590 | 340 |
|
75394 | 341 |
val start_date = Date.now() |
64140 | 342 |
|
77521
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
343 |
progress.echo( |
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
344 |
"Started at " + Build_Log.print_date(start_date) + |
77719 | 345 |
" (" + Isabelle_System.ml_identifier() + " on " + hostname(options) +")", |
77521
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
346 |
verbose = true) |
5642de4d225d
clarified signature: manage "verbose" flag via "progress";
wenzelm
parents:
77505
diff
changeset
|
347 |
progress.echo(Build_Log.Settings.show() + "\n", verbose = true) |
62590 | 348 |
|
75394 | 349 |
val results = |
350 |
progress.interrupt_handler { |
|
351 |
build(options, |
|
352 |
selection = Sessions.Selection( |
|
353 |
requirements = requirements, |
|
354 |
all_sessions = all_sessions, |
|
355 |
base_sessions = base_sessions, |
|
356 |
exclude_session_groups = exclude_session_groups, |
|
357 |
exclude_sessions = exclude_sessions, |
|
358 |
session_groups = session_groups, |
|
359 |
sessions = sessions), |
|
75942
603852abed8f
clarified names: Browser_Info.Config vs. Browser_Info.Context;
wenzelm
parents:
75941
diff
changeset
|
360 |
browser_info = browser_info, |
75394 | 361 |
progress = progress, |
362 |
check_unknown_files = Mercurial.is_repository(Path.ISABELLE_HOME), |
|
363 |
build_heap = build_heap, |
|
364 |
clean_build = clean_build, |
|
365 |
dirs = dirs, |
|
366 |
select_dirs = select_dirs, |
|
77477 | 367 |
numa_shuffling = Host.numa_check(progress, numa_shuffling), |
75394 | 368 |
max_jobs = max_jobs, |
369 |
list_files = list_files, |
|
370 |
check_keywords = check_keywords, |
|
371 |
fresh_build = fresh_build, |
|
372 |
no_build = no_build, |
|
373 |
soft_build = soft_build, |
|
374 |
export_files = export_files) |
|
375 |
} |
|
77545 | 376 |
val stop_date = Date.now() |
377 |
val elapsed_time = stop_date.time - start_date.time |
|
75394 | 378 |
|
77545 | 379 |
progress.echo("\nFinished at " + Build_Log.print_date(stop_date), verbose = true) |
62590 | 380 |
|
75394 | 381 |
val total_timing = |
382 |
results.sessions.iterator.map(a => results(a).timing).foldLeft(Timing.zero)(_ + _). |
|
383 |
copy(elapsed = elapsed_time) |
|
384 |
progress.echo(total_timing.message_resources) |
|
62590 | 385 |
|
75394 | 386 |
sys.exit(results.rc) |
387 |
}) |
|
68305 | 388 |
|
389 |
||
77553 | 390 |
|
77557 | 391 |
/** "isabelle build_worker" **/ |
392 |
||
78219 | 393 |
/* identified builds */ |
394 |
||
395 |
def read_builds(options: Options): List[Build_Process.Build] = |
|
78223 | 396 |
using_option(Store(options).maybe_open_build_database())( |
78222 | 397 |
Build_Process.read_builds).getOrElse(Nil).filter(_.active) |
78219 | 398 |
|
78221 | 399 |
def print_builds(options: Options, builds: List[Build_Process.Build]): String = |
78223 | 400 |
using_optional(Store(options).maybe_open_build_database()) { build_database => |
78221 | 401 |
val print_database = |
402 |
build_database match { |
|
403 |
case None => "" |
|
78225 | 404 |
case Some(db) => " (database: " + db + ")" |
78221 | 405 |
} |
406 |
if (builds.isEmpty) "No build processes available" + print_database |
|
407 |
else { |
|
78225 | 408 |
"Available build processes" + print_database + |
78221 | 409 |
(for ((build, i) <- builds.iterator.zipWithIndex) |
410 |
yield { |
|
411 |
"\n " + (i + 1) + ": " + build.build_uuid + |
|
412 |
" (platform: " + build.ml_platform + |
|
413 |
", start: " + Build_Log.print_date(build.start) + ")" |
|
414 |
}).mkString |
|
415 |
} |
|
78219 | 416 |
} |
417 |
||
78221 | 418 |
def id_builds( |
419 |
options: Options, |
|
420 |
id: String, |
|
421 |
builds: List[Build_Process.Build] |
|
422 |
): Build_Process.Build = |
|
78219 | 423 |
(id, builds.length) match { |
424 |
case (Value.Int(i), n) if 1 <= i && i <= n => builds(i - 1) |
|
425 |
case (UUID(_), _) if builds.exists(_.build_uuid == id) => builds.find(_.build_uuid == id).get |
|
78221 | 426 |
case ("", 0) => error(print_builds(options, builds)) |
78219 | 427 |
case ("", 1) => builds.head |
78221 | 428 |
case _ => cat_error("Cannot identify build process " + quote(id), print_builds(options, builds)) |
78219 | 429 |
} |
430 |
||
431 |
||
77557 | 432 |
/* build_worker */ |
433 |
||
434 |
def build_worker( |
|
435 |
options: Options, |
|
78219 | 436 |
build_master: Build_Process.Build, |
77557 | 437 |
progress: Progress = new Progress, |
438 |
dirs: List[Path] = Nil, |
|
439 |
numa_shuffling: Boolean = false, |
|
440 |
max_jobs: Int = 1, |
|
77559
4ad322ee6025
clarified signature: support all arguments of Sessions.store();
wenzelm
parents:
77558
diff
changeset
|
441 |
cache: Term.Cache = Term.Cache.make() |
77557 | 442 |
): Results = { |
78232 | 443 |
val build_engine = Engine(engine_name(options)) |
444 |
||
78233 | 445 |
val store = build_engine.build_store(options, cache = cache) |
77557 | 446 |
val build_options = store.options |
447 |
||
78219 | 448 |
val sessions_structure = |
449 |
Sessions.load_structure(build_options, dirs = dirs). |
|
78226 | 450 |
selection(Sessions.Selection(sessions = build_master.sessions)) |
78219 | 451 |
|
452 |
val build_deps = |
|
453 |
Sessions.deps(sessions_structure, progress = progress, inlined_files = true).check_errors |
|
454 |
||
455 |
val build_context = |
|
78237
c2c59de57df9
clarified static Build_Process.Context vs. dynamic Build_Process.State;
wenzelm
parents:
78233
diff
changeset
|
456 |
Build_Process.Context(store, build_deps, hostname = hostname(build_options), |
c2c59de57df9
clarified static Build_Process.Context vs. dynamic Build_Process.State;
wenzelm
parents:
78233
diff
changeset
|
457 |
numa_shuffling = numa_shuffling, max_jobs = max_jobs, build_uuid = build_master.build_uuid) |
78219 | 458 |
|
78232 | 459 |
build_engine.run(build_context, progress) |
77557 | 460 |
} |
461 |
||
462 |
||
463 |
/* command-line wrapper */ |
|
464 |
||
465 |
val isabelle_tool2 = Isabelle_Tool("build_worker", "external worker for session build process", |
|
466 |
Scala_Project.here, |
|
467 |
{ args => |
|
78219 | 468 |
var build_id = "" |
469 |
var list_builds = false |
|
77557 | 470 |
var numa_shuffling = false |
471 |
var dirs: List[Path] = Nil |
|
472 |
var max_jobs = 1 |
|
78219 | 473 |
var options = |
474 |
Options.init(specs = Options.Spec.ISABELLE_BUILD_OPTIONS ::: |
|
475 |
List(Options.Spec.make("build_database_test"))) |
|
77557 | 476 |
var verbose = false |
477 |
||
478 |
val getopts = Getopts(""" |
|
78219 | 479 |
Usage: isabelle build_worker [OPTIONS] |
77557 | 480 |
|
481 |
Options are: |
|
482 |
-N cyclic shuffling of NUMA CPU nodes (performance tuning) |
|
483 |
-d DIR include session directory |
|
78219 | 484 |
-i ID identify build process, either via index (starting from 1) or |
485 |
Universally Unique Identifier (UUID) |
|
77557 | 486 |
-j INT maximum number of parallel jobs (default 1) |
78219 | 487 |
-l list build processes |
77557 | 488 |
-o OPTION override Isabelle system OPTION (via NAME=VAL or NAME) |
489 |
-v verbose |
|
490 |
||
491 |
Run as external worker for session build process, as identified via |
|
78219 | 492 |
option -i. The latter can be omitted, if there is exactly one build. |
77647 | 493 |
""", |
77557 | 494 |
"N" -> (_ => numa_shuffling = true), |
495 |
"d:" -> (arg => dirs = dirs ::: List(Path.explode(arg))), |
|
78219 | 496 |
"i:" -> (arg => build_id = arg), |
77557 | 497 |
"j:" -> (arg => max_jobs = Value.Int.parse(arg)), |
78219 | 498 |
"l" -> (_ => list_builds = true), |
77557 | 499 |
"o:" -> (arg => options = options + arg), |
500 |
"v" -> (_ => verbose = true)) |
|
501 |
||
502 |
val more_args = getopts(args) |
|
503 |
if (more_args.nonEmpty) getopts.usage() |
|
504 |
||
505 |
val progress = new Console_Progress(verbose = verbose) |
|
506 |
||
78219 | 507 |
val builds = read_builds(options) |
508 |
||
78221 | 509 |
if (list_builds) progress.echo(print_builds(options, builds)) |
78219 | 510 |
|
511 |
if (!list_builds || build_id.nonEmpty) { |
|
78221 | 512 |
val build = id_builds(options, build_id, builds) |
77557 | 513 |
|
78219 | 514 |
val results = |
515 |
progress.interrupt_handler { |
|
516 |
build_worker(options, build, |
|
517 |
progress = progress, |
|
518 |
dirs = dirs, |
|
519 |
numa_shuffling = Host.numa_check(progress, numa_shuffling), |
|
520 |
max_jobs = max_jobs) |
|
521 |
} |
|
522 |
||
523 |
sys.exit(results.rc) |
|
524 |
} |
|
77557 | 525 |
}) |
526 |
||
527 |
||
528 |
||
77563 | 529 |
/** "isabelle build_log" **/ |
77553 | 530 |
|
531 |
/* theory markup/messages from session database */ |
|
532 |
||
533 |
def read_theory( |
|
534 |
theory_context: Export.Theory_Context, |
|
535 |
unicode_symbols: Boolean = false |
|
536 |
): Option[Document.Snapshot] = { |
|
537 |
def decode_bytes(bytes: Bytes): String = |
|
538 |
Symbol.output(unicode_symbols, UTF8.decode_permissive(bytes)) |
|
539 |
||
540 |
def read(name: String): Export.Entry = theory_context(name, permissive = true) |
|
541 |
||
542 |
def read_xml(name: String): XML.Body = |
|
543 |
YXML.parse_body(decode_bytes(read(name).bytes), cache = theory_context.cache) |
|
544 |
||
78178 | 545 |
def read_source_file(name: String): Store.Source_File = |
77553 | 546 |
theory_context.session_context.source_file(name) |
547 |
||
548 |
for { |
|
549 |
id <- theory_context.document_id() |
|
550 |
(thy_file, blobs_files) <- theory_context.files(permissive = true) |
|
551 |
} |
|
552 |
yield { |
|
553 |
val master_dir = |
|
554 |
Path.explode(Url.strip_base_name(thy_file).getOrElse( |
|
555 |
error("Cannot determine theory master directory: " + quote(thy_file)))) |
|
556 |
||
557 |
val blobs = |
|
558 |
blobs_files.map { name => |
|
559 |
val path = Path.explode(name) |
|
560 |
val src_path = File.relative_path(master_dir, path).getOrElse(path) |
|
561 |
||
562 |
val file = read_source_file(name) |
|
563 |
val bytes = file.bytes |
|
564 |
val text = decode_bytes(bytes) |
|
565 |
val chunk = Symbol.Text_Chunk(text) |
|
566 |
||
567 |
Command.Blob(Document.Node.Name(name), src_path, Some((file.digest, chunk))) -> |
|
568 |
Document.Blobs.Item(bytes, text, chunk, changed = false) |
|
569 |
} |
|
570 |
||
571 |
val thy_source = decode_bytes(read_source_file(thy_file).bytes) |
|
572 |
val thy_xml = read_xml(Export.MARKUP) |
|
573 |
val blobs_xml = |
|
574 |
for (i <- (1 to blobs.length).toList) |
|
575 |
yield read_xml(Export.MARKUP + i) |
|
576 |
||
577 |
val markups_index = Command.Markup_Index.make(blobs.map(_._1)) |
|
578 |
val markups = |
|
579 |
Command.Markups.make( |
|
580 |
for ((index, xml) <- markups_index.zip(thy_xml :: blobs_xml)) |
|
581 |
yield index -> Markup_Tree.from_XML(xml)) |
|
582 |
||
583 |
val results = |
|
584 |
Command.Results.make( |
|
585 |
for (elem @ XML.Elem(Markup(_, Markup.Serial(i)), _) <- read_xml(Export.MESSAGES)) |
|
586 |
yield i -> elem) |
|
587 |
||
588 |
val command = |
|
589 |
Command.unparsed(thy_source, theory = true, id = id, |
|
590 |
node_name = Document.Node.Name(thy_file, theory = theory_context.theory), |
|
591 |
blobs_info = Command.Blobs_Info.make(blobs), |
|
592 |
markups = markups, results = results) |
|
593 |
||
594 |
val doc_blobs = Document.Blobs.make(blobs) |
|
595 |
||
596 |
Document.State.init.snippet(command, doc_blobs) |
|
597 |
} |
|
598 |
} |
|
599 |
||
600 |
||
601 |
/* print messages */ |
|
602 |
||
603 |
def print_log( |
|
604 |
options: Options, |
|
605 |
sessions: List[String], |
|
606 |
theories: List[String] = Nil, |
|
607 |
message_head: List[Regex] = Nil, |
|
608 |
message_body: List[Regex] = Nil, |
|
609 |
progress: Progress = new Progress, |
|
610 |
margin: Double = Pretty.default_margin, |
|
611 |
breakgain: Double = Pretty.default_breakgain, |
|
612 |
metric: Pretty.Metric = Symbol.Metric, |
|
613 |
unicode_symbols: Boolean = false |
|
614 |
): Unit = { |
|
78178 | 615 |
val store = Store(options) |
77553 | 616 |
val session = new Session(options, Resources.bootstrap) |
617 |
||
618 |
def check(filter: List[Regex], make_string: => String): Boolean = |
|
619 |
filter.isEmpty || { |
|
620 |
val s = Output.clean_yxml(make_string) |
|
621 |
filter.forall(r => r.findFirstIn(Output.clean_yxml(s)).nonEmpty) |
|
622 |
} |
|
623 |
||
624 |
def print(session_name: String): Unit = { |
|
625 |
using(Export.open_session_context0(store, session_name)) { session_context => |
|
626 |
val result = |
|
627 |
for { |
|
628 |
db <- session_context.session_db() |
|
629 |
theories = store.read_theories(db, session_name) |
|
630 |
errors = store.read_errors(db, session_name) |
|
631 |
info <- store.read_build(db, session_name) |
|
632 |
} yield (theories, errors, info.return_code) |
|
633 |
result match { |
|
634 |
case None => store.error_database(session_name) |
|
635 |
case Some((used_theories, errors, rc)) => |
|
636 |
theories.filterNot(used_theories.toSet) match { |
|
637 |
case Nil => |
|
638 |
case bad => error("Unknown theories " + commas_quote(bad)) |
|
639 |
} |
|
640 |
val print_theories = |
|
641 |
if (theories.isEmpty) used_theories else used_theories.filter(theories.toSet) |
|
642 |
||
643 |
for (thy <- print_theories) { |
|
644 |
val thy_heading = "\nTheory " + quote(thy) + " (in " + session_name + ")" + ":" |
|
645 |
||
646 |
Build_Job.read_theory(session_context.theory(thy), unicode_symbols = unicode_symbols) match { |
|
647 |
case None => progress.echo(thy_heading + " MISSING") |
|
648 |
case Some(snapshot) => |
|
649 |
val rendering = new Rendering(snapshot, options, session) |
|
650 |
val messages = |
|
651 |
rendering.text_messages(Text.Range.full) |
|
652 |
.filter(message => progress.verbose || Protocol.is_exported(message.info)) |
|
653 |
if (messages.nonEmpty) { |
|
654 |
val line_document = Line.Document(snapshot.node.source) |
|
655 |
val buffer = new mutable.ListBuffer[String] |
|
656 |
for (Text.Info(range, elem) <- messages) { |
|
657 |
val line = line_document.position(range.start).line1 |
|
658 |
val pos = Position.Line_File(line, snapshot.node_name.node) |
|
659 |
def message_text: String = |
|
660 |
Protocol.message_text(elem, heading = true, pos = pos, |
|
661 |
margin = margin, breakgain = breakgain, metric = metric) |
|
662 |
val ok = |
|
663 |
check(message_head, Protocol.message_heading(elem, pos)) && |
|
664 |
check(message_body, XML.content(Pretty.unformatted(List(elem)))) |
|
665 |
if (ok) buffer += message_text |
|
666 |
} |
|
667 |
if (buffer.nonEmpty) { |
|
668 |
progress.echo(thy_heading) |
|
669 |
buffer.foreach(progress.echo(_)) |
|
670 |
} |
|
671 |
} |
|
672 |
} |
|
673 |
} |
|
674 |
||
675 |
if (errors.nonEmpty) { |
|
676 |
val msg = Symbol.output(unicode_symbols, cat_lines(errors)) |
|
677 |
progress.echo("\nBuild errors:\n" + Output.error_message_text(msg)) |
|
678 |
} |
|
679 |
if (rc != Process_Result.RC.ok) { |
|
680 |
progress.echo("\n" + Process_Result.RC.print_long(rc)) |
|
681 |
} |
|
682 |
} |
|
683 |
} |
|
684 |
} |
|
685 |
||
686 |
val errors = new mutable.ListBuffer[String] |
|
687 |
for (session_name <- sessions) { |
|
688 |
Exn.interruptible_capture(print(session_name)) match { |
|
689 |
case Exn.Res(_) => |
|
690 |
case Exn.Exn(exn) => errors += Exn.message(exn) |
|
691 |
} |
|
692 |
} |
|
693 |
if (errors.nonEmpty) error(cat_lines(errors.toList)) |
|
694 |
} |
|
695 |
||
696 |
||
697 |
/* command-line wrapper */ |
|
698 |
||
77563 | 699 |
val isabelle_tool3 = Isabelle_Tool("build_log", "print messages from session build database", |
77553 | 700 |
Scala_Project.here, |
701 |
{ args => |
|
702 |
/* arguments */ |
|
703 |
||
704 |
var message_head = List.empty[Regex] |
|
705 |
var message_body = List.empty[Regex] |
|
706 |
var unicode_symbols = false |
|
707 |
var theories: List[String] = Nil |
|
708 |
var margin = Pretty.default_margin |
|
709 |
var options = Options.init() |
|
710 |
var verbose = false |
|
711 |
||
712 |
val getopts = Getopts(""" |
|
77563 | 713 |
Usage: isabelle build_log [OPTIONS] [SESSIONS ...] |
77553 | 714 |
|
715 |
Options are: |
|
716 |
-H REGEX filter messages by matching against head |
|
717 |
-M REGEX filter messages by matching against body |
|
718 |
-T NAME restrict to given theories (multiple options possible) |
|
719 |
-U output Unicode symbols |
|
720 |
-m MARGIN margin for pretty printing (default: """ + margin + """) |
|
721 |
-o OPTION override Isabelle system OPTION (via NAME=VAL or NAME) |
|
722 |
-v print all messages, including information etc. |
|
723 |
||
77554
4465d9dff448
clarified terminology of "session build database", while "build database" is the one underlying Build_Process;
wenzelm
parents:
77553
diff
changeset
|
724 |
Print messages from the session build database of the given sessions, |
4465d9dff448
clarified terminology of "session build database", while "build database" is the one underlying Build_Process;
wenzelm
parents:
77553
diff
changeset
|
725 |
without any checks against current sources nor session structure: results |
4465d9dff448
clarified terminology of "session build database", while "build database" is the one underlying Build_Process;
wenzelm
parents:
77553
diff
changeset
|
726 |
from old sessions or failed builds can be printed as well. |
77553 | 727 |
|
728 |
Multiple options -H and -M are conjunctive: all given patterns need to |
|
729 |
match. Patterns match any substring, but ^ or $ may be used to match the |
|
730 |
start or end explicitly. |
|
731 |
""", |
|
732 |
"H:" -> (arg => message_head = message_head ::: List(arg.r)), |
|
733 |
"M:" -> (arg => message_body = message_body ::: List(arg.r)), |
|
734 |
"T:" -> (arg => theories = theories ::: List(arg)), |
|
735 |
"U" -> (_ => unicode_symbols = true), |
|
736 |
"m:" -> (arg => margin = Value.Double.parse(arg)), |
|
737 |
"o:" -> (arg => options = options + arg), |
|
738 |
"v" -> (_ => verbose = true)) |
|
739 |
||
740 |
val sessions = getopts(args) |
|
741 |
||
742 |
val progress = new Console_Progress(verbose = verbose) |
|
743 |
||
744 |
if (sessions.isEmpty) progress.echo_warning("No sessions to print") |
|
745 |
else { |
|
746 |
print_log(options, sessions, theories = theories, message_head = message_head, |
|
747 |
message_body = message_body, margin = margin, progress = progress, |
|
748 |
unicode_symbols = unicode_symbols) |
|
749 |
} |
|
750 |
}) |
|
48276 | 751 |
} |