2021-12-15 08:24:49 +00:00
|
|
|
/-
|
|
|
|
Copyright (c) 2021 Henrik Böving. All rights reserved.
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
Authors: Henrik Böving
|
|
|
|
-/
|
|
|
|
import DocGen4.Output.Template
|
2022-01-03 17:22:12 +00:00
|
|
|
import DocGen4.Output.Inductive
|
2022-01-04 07:23:39 +00:00
|
|
|
import DocGen4.Output.Structure
|
2022-01-06 13:28:41 +00:00
|
|
|
import DocGen4.Output.Class
|
2022-02-02 10:22:15 +00:00
|
|
|
import DocGen4.Output.Definition
|
2022-02-04 21:48:08 +00:00
|
|
|
import DocGen4.Output.Instance
|
2022-02-06 19:14:36 +00:00
|
|
|
import DocGen4.Output.ClassInductive
|
2022-02-17 05:47:38 +00:00
|
|
|
import DocGen4.Output.DocString
|
2022-05-19 22:36:43 +00:00
|
|
|
import DocGen4.Process
|
2022-02-15 18:19:40 +00:00
|
|
|
import Lean.Data.Xml.Parser
|
2021-12-15 08:24:49 +00:00
|
|
|
|
|
|
|
namespace DocGen4
|
|
|
|
namespace Output
|
|
|
|
|
|
|
|
open scoped DocGen4.Jsx
|
2022-05-19 22:36:43 +00:00
|
|
|
open Lean Process
|
2021-12-25 13:08:09 +00:00
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Render an `Arg` as HTML, adding opacity effects etc. depending on what
|
|
|
|
type of binder it has.
|
|
|
|
-/
|
2021-12-25 15:55:30 +00:00
|
|
|
def argToHtml (arg : Arg) : HtmlM Html := do
|
|
|
|
let (l, r, implicit) := match arg.binderInfo with
|
|
|
|
| BinderInfo.default => ("(", ")", false)
|
|
|
|
| BinderInfo.implicit => ("{", "}", true)
|
|
|
|
| BinderInfo.strictImplicit => ("⦃", "⦄", true)
|
|
|
|
| BinderInfo.instImplicit => ("[", "]", true)
|
|
|
|
let mut nodes := #[Html.text s!"{l}{arg.name.toString} : "]
|
|
|
|
nodes := nodes.append (←infoFormatToHtml arg.type)
|
|
|
|
nodes := nodes.push r
|
2022-06-21 18:54:29 +00:00
|
|
|
let inner := <span class="fn">[nodes]</span>
|
2021-12-25 15:55:30 +00:00
|
|
|
let html := Html.element "span" false #[("class", "decl_args")] #[inner]
|
|
|
|
if implicit then
|
2022-05-19 09:14:47 +00:00
|
|
|
pure <span class="impl_arg">{html}</span>
|
2021-12-25 15:55:30 +00:00
|
|
|
else
|
2022-02-12 14:09:13 +00:00
|
|
|
pure html
|
2021-12-25 15:55:30 +00:00
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Render the structures this structure extends from as HTML so it can be
|
|
|
|
added to the top level.
|
|
|
|
-/
|
2022-05-19 22:36:43 +00:00
|
|
|
def structureInfoHeader (s : Process.StructureInfo) : HtmlM (Array Html) := do
|
2022-01-04 07:23:39 +00:00
|
|
|
let mut nodes := #[]
|
|
|
|
if s.parents.size > 0 then
|
2022-05-19 09:14:47 +00:00
|
|
|
nodes := nodes.push <span class="decl_extends">extends</span>
|
2022-01-04 07:23:39 +00:00
|
|
|
let mut parents := #[]
|
|
|
|
for parent in s.parents do
|
2022-05-19 19:40:22 +00:00
|
|
|
let link ← declNameToHtmlBreakWithinLink parent
|
2022-06-21 18:54:29 +00:00
|
|
|
let inner := <span class="fn">{link}</span>
|
2022-01-04 07:23:39 +00:00
|
|
|
let html:= Html.element "span" false #[("class", "decl_parent")] #[inner]
|
|
|
|
parents := parents.push html
|
|
|
|
nodes := nodes.append (parents.toList.intersperse (Html.text ", ")).toArray
|
2022-02-12 14:09:13 +00:00
|
|
|
pure nodes
|
2022-01-04 07:23:39 +00:00
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Render the general header of a declaration containing its declaration type
|
|
|
|
and name.
|
|
|
|
-/
|
2021-12-17 14:59:43 +00:00
|
|
|
def docInfoHeader (doc : DocInfo) : HtmlM Html := do
|
|
|
|
let mut nodes := #[]
|
2022-07-23 11:01:25 +00:00
|
|
|
nodes := nodes.push <| Html.element "span" false #[("class", "decl_kind")] #[doc.getKindDescription]
|
2021-12-17 16:20:44 +00:00
|
|
|
nodes := nodes.push
|
2022-05-19 09:14:47 +00:00
|
|
|
<span class="decl_name">
|
|
|
|
<a class="break_within" href={←declNameToLink doc.getName}>
|
2021-12-17 16:20:44 +00:00
|
|
|
-- TODO: HTMLify the name
|
|
|
|
{doc.getName.toString}
|
|
|
|
</a>
|
|
|
|
</span>
|
2021-12-25 15:55:30 +00:00
|
|
|
for arg in doc.getArgs do
|
|
|
|
nodes := nodes.push (←argToHtml arg)
|
2022-01-04 07:23:39 +00:00
|
|
|
|
2022-01-06 13:28:41 +00:00
|
|
|
match doc with
|
|
|
|
| DocInfo.structureInfo i => nodes := nodes.append (←structureInfoHeader i)
|
2022-07-22 12:48:36 +00:00
|
|
|
| DocInfo.classInfo i => nodes := nodes.append (←structureInfoHeader i)
|
2022-01-06 13:28:41 +00:00
|
|
|
| _ => nodes := nodes
|
2022-01-04 07:23:39 +00:00
|
|
|
|
2022-07-27 12:19:40 +00:00
|
|
|
nodes := nodes.push <| Html.element "span" true #[("class", "decl_args")] #[" :"]
|
2022-06-21 18:54:29 +00:00
|
|
|
nodes := nodes.push <div class="decl_type">[←infoFormatToHtml doc.getType]</div>
|
2022-05-19 09:14:47 +00:00
|
|
|
pure <div class="decl_header"> [nodes] </div>
|
2021-12-15 08:24:49 +00:00
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
The main entry point for rendering a single declaration inside a given module.
|
|
|
|
-/
|
2022-01-09 15:57:19 +00:00
|
|
|
def docInfoToHtml (module : Name) (doc : DocInfo) : HtmlM Html := do
|
2022-02-19 19:14:58 +00:00
|
|
|
-- basic info like headers, types, structure fields, etc.
|
2022-02-18 03:28:44 +00:00
|
|
|
let docInfoHtml ← match doc with
|
2022-01-03 17:22:12 +00:00
|
|
|
| DocInfo.inductiveInfo i => inductiveToHtml i
|
2022-01-04 07:23:39 +00:00
|
|
|
| DocInfo.structureInfo i => structureToHtml i
|
2022-01-06 13:28:41 +00:00
|
|
|
| DocInfo.classInfo i => classToHtml i
|
2022-02-06 19:14:36 +00:00
|
|
|
| DocInfo.classInductiveInfo i => classInductiveToHtml i
|
2022-07-22 12:48:36 +00:00
|
|
|
| _ => pure #[]
|
2022-02-19 19:14:58 +00:00
|
|
|
-- rendered doc stirng
|
2022-02-18 03:28:44 +00:00
|
|
|
let docStringHtml ← match doc.getDocString with
|
|
|
|
| some s => docStringToHtml s
|
|
|
|
| none => pure #[]
|
2022-02-19 19:14:58 +00:00
|
|
|
-- extra information like equations and instances
|
|
|
|
let extraInfoHtml ← match doc with
|
2022-07-22 12:48:36 +00:00
|
|
|
| DocInfo.classInfo i => pure #[←classInstancesToHtml i.name]
|
2022-02-19 19:14:58 +00:00
|
|
|
| DocInfo.definitionInfo i => equationsToHtml i
|
2022-07-22 12:48:36 +00:00
|
|
|
| DocInfo.instanceInfo i => equationsToHtml i.toDefinitionInfo
|
|
|
|
| DocInfo.classInductiveInfo i => pure #[←classInstancesToHtml i.name]
|
2022-07-23 13:40:08 +00:00
|
|
|
| DocInfo.inductiveInfo i => pure #[←instancesForToHtml i.name]
|
|
|
|
| DocInfo.structureInfo i => pure #[←instancesForToHtml i.name]
|
2022-07-22 12:48:36 +00:00
|
|
|
| _ => pure #[]
|
2022-02-13 02:32:53 +00:00
|
|
|
let attrs := doc.getAttrs
|
|
|
|
let attrsHtml :=
|
|
|
|
if attrs.size > 0 then
|
|
|
|
let attrStr := "@[" ++ String.intercalate ", " doc.getAttrs.toList ++ "]"
|
|
|
|
#[Html.element "div" false #[("class", "attributes")] #[attrStr]]
|
|
|
|
else
|
|
|
|
#[]
|
2022-06-19 22:31:09 +00:00
|
|
|
let leanInkHtml :=
|
|
|
|
if ←leanInkEnabled? then
|
|
|
|
#[
|
|
|
|
<div class="ink_link">
|
|
|
|
<a href={←declNameToInkLink doc.getName}>ink</a>
|
|
|
|
</div>
|
|
|
|
]
|
|
|
|
else
|
|
|
|
#[]
|
2022-02-13 02:32:53 +00:00
|
|
|
|
2022-02-12 14:09:13 +00:00
|
|
|
pure
|
2022-05-19 09:14:47 +00:00
|
|
|
<div class="decl" id={doc.getName.toString}>
|
|
|
|
<div class={doc.getKind}>
|
|
|
|
<div class="gh_link">
|
2022-02-12 14:09:13 +00:00
|
|
|
<a href={←getSourceUrl module doc.getDeclarationRange}>source</a>
|
|
|
|
</div>
|
2022-06-19 22:31:09 +00:00
|
|
|
[leanInkHtml]
|
2022-02-13 02:32:53 +00:00
|
|
|
[attrsHtml]
|
2022-02-12 14:09:13 +00:00
|
|
|
{←docInfoHeader doc}
|
2022-02-18 03:28:44 +00:00
|
|
|
[docInfoHtml]
|
2022-02-19 19:14:58 +00:00
|
|
|
[docStringHtml]
|
|
|
|
[extraInfoHtml]
|
2021-12-15 10:59:36 +00:00
|
|
|
</div>
|
|
|
|
</div>
|
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Rendering a module doc string, that is the ones with an ! after the opener
|
|
|
|
as HTML.
|
|
|
|
-/
|
2022-07-22 12:48:36 +00:00
|
|
|
def modDocToHtml (mdoc : ModuleDoc) : HtmlM Html := do
|
2022-10-20 17:51:26 +00:00
|
|
|
pure
|
2022-05-19 09:14:47 +00:00
|
|
|
<div class="mod_doc">
|
2022-02-17 13:26:02 +00:00
|
|
|
[←docStringToHtml mdoc.doc]
|
2022-02-15 17:06:46 +00:00
|
|
|
</div>
|
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Render a module member, that is either a module doc string or a declaration
|
|
|
|
as HTML.
|
|
|
|
-/
|
2022-02-18 03:28:44 +00:00
|
|
|
def moduleMemberToHtml (module : Name) (member : ModuleMember) : HtmlM Html := do
|
2022-02-15 17:06:46 +00:00
|
|
|
match member with
|
|
|
|
| ModuleMember.docInfo d => docInfoToHtml module d
|
2022-07-22 12:48:36 +00:00
|
|
|
| ModuleMember.modDoc d => modDocToHtml d
|
2022-02-15 17:06:46 +00:00
|
|
|
|
2022-01-16 13:22:53 +00:00
|
|
|
def declarationToNavLink (module : Name) : Html :=
|
2022-05-19 09:14:47 +00:00
|
|
|
<div class="nav_link">
|
|
|
|
<a class="break_within" href={s!"#{module.toString}"}>{module.toString}</a>
|
2022-01-07 16:43:49 +00:00
|
|
|
</div>
|
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Returns the list of all imports this module does.
|
|
|
|
-/
|
2022-01-16 13:22:53 +00:00
|
|
|
def getImports (module : Name) : HtmlM (Array Name) := do
|
|
|
|
let res ← getResult
|
2022-07-23 11:01:25 +00:00
|
|
|
pure <| res.moduleInfo.find! module |>.imports
|
2022-01-16 13:22:53 +00:00
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
Sort the list of all modules this one is importing, linkify it
|
|
|
|
and return the HTML.
|
|
|
|
-/
|
|
|
|
def importsHtml (moduleName : Name) : HtmlM (Array Html) := do
|
|
|
|
let imports := (←getImports moduleName) |>.qsort Name.lt
|
|
|
|
imports.mapM (λ i => do pure <li>{←moduleToHtmlLink i}</li>)
|
|
|
|
|
|
|
|
/--
|
|
|
|
Render the internal nav bar (the thing on the right on all module pages).
|
|
|
|
-/
|
2022-01-09 15:57:19 +00:00
|
|
|
def internalNav (members : Array Name) (moduleName : Name) : HtmlM Html := do
|
2022-02-12 14:09:13 +00:00
|
|
|
pure
|
2022-05-19 09:14:47 +00:00
|
|
|
<nav class="internal_nav">
|
|
|
|
<h3><a class="break_within" href="#top">{moduleName.toString}</a></h3>
|
|
|
|
<p class="gh_nav_link"><a href={←getSourceUrl moduleName none}>source</a></p>
|
|
|
|
<div class="imports">
|
2022-02-12 14:09:13 +00:00
|
|
|
<details>
|
|
|
|
<summary>Imports</summary>
|
|
|
|
<ul>
|
|
|
|
[←importsHtml moduleName]
|
|
|
|
</ul>
|
|
|
|
</details>
|
|
|
|
<details>
|
|
|
|
<summary>Imported by</summary>
|
2022-07-22 14:56:51 +00:00
|
|
|
<ul id={s!"imported-by-{moduleName}"} class="imported-by-list"> </ul>
|
2022-02-12 14:09:13 +00:00
|
|
|
</details>
|
|
|
|
</div>
|
|
|
|
[members.map declarationToNavLink]
|
|
|
|
</nav>
|
2022-01-07 16:43:49 +00:00
|
|
|
|
2022-05-19 19:40:22 +00:00
|
|
|
/--
|
|
|
|
The main entry point to rendering the HTML for an entire module.
|
|
|
|
-/
|
2022-07-20 23:40:04 +00:00
|
|
|
def moduleToHtml (module : Process.Module) : HtmlM Html := withTheReader SiteBaseContext (setCurrentName module.name) do
|
2022-02-18 04:52:01 +00:00
|
|
|
let memberDocs ← module.members.mapM (λ i => moduleMemberToHtml module.name i)
|
|
|
|
let memberNames := filterMapDocInfo module.members |>.map DocInfo.getName
|
2022-07-23 11:01:25 +00:00
|
|
|
templateLiftExtends (baseHtmlGenerator module.name.toString) <| pure #[
|
2022-02-18 04:52:01 +00:00
|
|
|
←internalNav memberNames module.name,
|
|
|
|
Html.element "main" false #[] memberDocs
|
2022-01-07 16:43:49 +00:00
|
|
|
]
|
2021-12-15 08:24:49 +00:00
|
|
|
|
|
|
|
end Output
|
|
|
|
end DocGen4
|