diff -r cbae5c5ffd23 -r d90218288d51 src/Tools/WWW_Find/Start_WWW_Find.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/Tools/WWW_Find/Start_WWW_Find.thy Mon Feb 11 14:39:04 2013 +0100 @@ -0,0 +1,14 @@ +(* 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 +