src/Tools/WWW_Find/Start_WWW_Find.thy
changeset 51950 13fb5e4f2893
parent 51949 f6858bb224c9
child 51979 4f3a5f4c1169
equal deleted inserted replaced
51949:f6858bb224c9 51950:13fb5e4f2893
     5 theory Start_WWW_Find imports WWW_Find begin
     5 theory Start_WWW_Find imports WWW_Find begin
     6 
     6 
     7 ML {*
     7 ML {*
     8   Options.default_put_bool "show_question_marks" false;
     8   Options.default_put_bool "show_question_marks" false;
     9   YXML_Find_Theorems.init ();
     9   YXML_Find_Theorems.init ();
    10   val port = OS.Process.getEnv "SCGIPORT" |> the |> Int.fromString |> the;
    10   val port = Markup.parse_int (getenv "SCGIPORT");
    11   ScgiServer.server' 10 "/" port;
    11   ScgiServer.server' 10 "/" port;
    12 *}
    12 *}
    13 
    13 
    14 end
    14 end
    15 
    15