/- 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 import DocGen4.Output.Inductive import DocGen4.Output.Structure import DocGen4.Output.Class namespace DocGen4 namespace Output open scoped DocGen4.Jsx open Lean 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) -- TODO: Can this ever be reached here? What does it mean? | BinderInfo.auxDecl => unreachable! let mut nodes := #[Html.text s!"{l}{arg.name.toString} : "] nodes := nodes.append (←infoFormatToHtml arg.type) nodes := nodes.push r let inner := Html.element "span" true #[("class", "fn")] nodes let html := Html.element "span" false #[("class", "decl_args")] #[inner] if implicit then {html} else html def structureInfoHeader (s : StructureInfo) : HtmlM (Array Html) := do let mut nodes := #[] if s.parents.size > 0 then nodes := nodes.push extends let mut parents := #[] for parent in s.parents do let link := {parent.toString} let inner := Html.element "span" true #[("class", "fn")] #[link] let html:= Html.element "span" false #[("class", "decl_parent")] #[inner] parents := parents.push html nodes := nodes.append (parents.toList.intersperse (Html.text ", ")).toArray nodes def docInfoHeader (doc : DocInfo) : HtmlM Html := do let mut nodes := #[] -- TODO: noncomputable, partial -- TODO: Support all the kinds in CSS nodes := nodes.push {doc.getKind} nodes := nodes.push -- TODO: HTMLify the name {doc.getName.toString} for arg in doc.getArgs do nodes := nodes.push (←argToHtml arg) -- TODO: dedup this match doc with | DocInfo.structureInfo i => nodes := nodes.append (←structureInfoHeader i) | DocInfo.classInfo i => nodes := nodes.append (←structureInfoHeader i.toStructureInfo) | _ => nodes := nodes nodes := nodes.push : nodes := nodes.push $ Html.element "div" true #[("class", "decl_type")] (←infoFormatToHtml doc.getType) return
[nodes]
def docInfoToHtml (doc : DocInfo) : HtmlM Html := do let doc_html ← match doc with | DocInfo.inductiveInfo i => inductiveToHtml i | DocInfo.structureInfo i => structureToHtml i | DocInfo.classInfo i => classToHtml i | _ => #[] return
-- TODO: Put the proper source link source
-- TODO: Attributes {←docInfoHeader doc} [←doc_html]
def moduleToNavLink (module : Name) : Html :=
{module.toString}
def internalNav (members : Array Name) (moduleName : Name) : Html := def moduleToHtml (module : Module) : HtmlM Html := withReader (setCurrentName module.name) do let docInfos ← module.members.mapM docInfoToHtml -- TODO: This is missing imports, imported by templateExtends (baseHtmlArray module.name.toString) $ #[ internalNav (module.members.map DocInfo.getName) module.name, Html.element "main" false #[] docInfos ] end Output end DocGen4