author | wenzelm |
Mon, 11 Feb 2013 14:39:04 +0100 | |
changeset 51085 | d90218288d51 |
child 51949 | f6858bb224c9 |
permissions | -rw-r--r-- |
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 (); |
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
|
9 |
val port = OS.Process.getEnv "SCGIPORT" |> the |> Int.fromString |> the; |
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 |