| author | wenzelm |
| Thu, 01 Aug 2013 22:19:32 +0200 | |
| changeset 52834 | a3f8c9f16d26 |
| parent 52057 | 69137d20ab0b |
| child 52926 | 6415d95bf7a2 |
| permissions | -rw-r--r-- |
(* 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 = Markup.parse_int (getenv "SCGIPORT"); ScgiServer.server' 10 "/" port; *} end