src/Tools/WWW_Find/Start_WWW_Find.thy
author wenzelm
Wed, 03 Apr 2013 21:30:32 +0200
changeset 51605 eca8acb42e4a
parent 51085 d90218288d51
child 51949 f6858bb224c9
permissions -rw-r--r--
more explicit Goal.fork_params -- avoid implicit arguments via thread data; actually fork terminal proofs in interactive mode (amending 8707df0b0255);

(* 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 {*
  YXML_Find_Theorems.init ();
  val port = OS.Process.getEnv "SCGIPORT" |> the |> Int.fromString |> the;
  ScgiServer.server' 10 "/" port;
*}

end