some secondary shortcuts derived from 5.1.0/keymaps/German_Keyboard_keys.props (using CIRCUMFLEX instead of S+1);
tuned;
(* 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