src/Tools/WWW_Find/Start_WWW_Find.thy
author wenzelm
Mon, 27 May 2013 22:26:08 +0200
changeset 52190 c87b7f26e2c7
parent 52057 69137d20ab0b
child 52926 6415d95bf7a2
permissions -rw-r--r--
merged
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
51085
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     1
(* Load this theory to start the WWW_Find server on port defined by environment
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     2
   variable "SCGIPORT". Used by the isabelle wwwfind tool.
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     3
*)
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     4
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     5
theory Start_WWW_Find imports WWW_Find begin
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     6
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     7
ML {*
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
     8
  YXML_Find_Theorems.init ();
51950
13fb5e4f2893 prefer standard Isabelle/ML operations;
wenzelm
parents: 51949
diff changeset
     9
  val port = Markup.parse_int (getenv "SCGIPORT");
51085
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
    10
  ScgiServer.server' 10 "/" port;
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
    11
*}
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
    12
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
    13
end
d90218288d51 make WWW_Find work again, now that its ML modules reside within a theory context (cf. bf5b45870110) -- patch by Rafal Kolanski;
wenzelm
parents:
diff changeset
    14