some rephrasing to ensure that this becomes cheap "foreach" and not expensive "map" (cf. 0fc032898b05);
(* Load this theory to start the WWW_Find server on port defined by environment
variable "SCGIPORT". Used by the isabelle wwwfind tool.
*)
theory Start_WWW_Find imports WWW_Find begin
ML {*
val port = Markup.parse_int (getenv "SCGIPORT");
ScgiServer.server' 10 "/" port;
*}
end