diff -r 0f22f7b370b2 -r 1be62b17bed9 src/Doc/System/Presentation.thy --- a/src/Doc/System/Presentation.thy Sun Feb 02 14:16:26 2025 +0100 +++ b/src/Doc/System/Presentation.thy Sun Feb 02 16:04:09 2025 +0100 @@ -208,14 +208,13 @@ text \ The session information of a regular @{tool_ref build} can also be used to generate a search index for full-text search over formal theory content. To - that end, the \<^verbatim>\Find_Facts\ module integrates Apache Solr\<^footnote>\\<^url>\https://solr.apache.org/\\, + that end, the \<^verbatim>\Find_Facts\ module integrates Apache Solr\<^footnote>\\<^url>\https://solr.apache.org\\, a full-text search engine, that can run embedded in a JVM process. Solr is bundled as a separate Isabelle component, and its run-time dependencies (as specified in @{setting SOLR_JARS}) need to be added separately to the classpath of a regular Isabelle/Scala process. \<^medskip> - A search index can be created using the @{tool_def find_facts_index} tool, which has options similar to the regular @{tool_ref build}. User data such as search indexes is stored in @{setting FIND_FACTS_HOME_USER}. The name of @@ -242,19 +241,19 @@ \} This Isabelle/Scala HTTP server provides the both the front-end - (implemented in the Elm\<^footnote>\\<^url>\https://elm-lang.org/\\ language) and REST + (implemented in the Elm\<^footnote>\\<^url>\https://elm-lang.org\\ language) and REST endpoints for search queries with JSON data. - Options \<^verbatim>\-o\, \-v\ have the same meaning as usual. + Options \<^verbatim>\-o\ and \<^verbatim>\-v\ have the same meaning as in @{tool build}. Option \<^verbatim>\-d\ re-compiles the front-end in \<^path>\$FIND_FACTS_HOME_USER/web\ on page reload (when sources are changed). - Option \<^verbatim>\-p\ specifies an explicit TCP port for the server socket - (assigned by the operating system per default). For public-facing servers, - a common scheme is \<^verbatim>\-p 8080\ that is access-restricted via firewall rules, - with a reverse proxy in system space (that also handles SSL) on ports 80 and - 443. + Option \<^verbatim>\-p\ specifies an explicit TCP port for the server socket (assigned + by the operating system per default). For public-facing servers, a common + scheme is \<^verbatim>\-p 8080\ that is access-restricted via firewall rules, with a + reverse proxy\<^footnote>\E.g. via Caddy \<^url>\https://caddyserver.com/docs\\ in system + space (that also handles SSL) on ports 80 and 443. \ end