/- 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 Lean import Lean.PrettyPrinter import DocGen4.ToHtmlFormat import DocGen4.Output.Template namespace DocGen4 namespace Output open scoped DocGen4.Jsx open Lean PrettyPrinter 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} -- TODO: HTMLify the name etc. nodes := nodes.push doc.getName.toString -- TODO: Figure out how we can get explicit, implicit and TC args and put them here nodes := nodes.push : nodes := nodes.push
Type!!!
-- TODO: The final type of the declaration return
[nodes]
def docInfoToHtml (doc : DocInfo) : HtmlM Html := do
-- TODO: Put the proper source link source
-- TODO: Attributes {←docInfoHeader doc} -- TODO: The actual type information we are here for
def moduleToHtml (module : Module) : HtmlM Html := withReader (setCurrentName module.name) do -- TODO: Probably some sort of ordering by line number would be cool? -- maybe they should already be ordered in members. let docInfos ← module.members.mapM docInfoToHtml -- TODO: This is missing imports, imported by, source link, list of decls templateExtends (baseHtml module.name.toString) $ Html.element "main" #[] docInfos end Output end DocGen4