/- 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 declNameToLink (name : Name) : HtmlM String := do let res ← getResult let module := res.moduleNames[res.name2ModIdx.find! name] (←moduleNameToLink module) ++ "#" ++ name.toString 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} -- TODO: Figure out how we can get explicit, implicit and TC args and put them here nodes := nodes.push : nodes := nodes.push