/- 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 DocGen4.ToHtmlFormat import DocGen4.Output.Base namespace DocGen4 namespace Output open Lean open scoped DocGen4.Jsx def moduleListFile (file : Name) : HtmlM Html := do let attributes := match ←getCurrentName with | some name => if file == name then #[("class", "nav_link"), ("visible", "")] else #[("class", "nav_link")] | none => #[("class", "nav_link")] let nodes := #[{file.toString}] return Html.element "div" attributes nodes partial def moduleListDir (h : Hierarchy) : HtmlM Html := do let children := Array.mk (h.getChildren.toList.map Prod.snd) let dirs := children.filter (λ c => c.getChildren.toList.length != 0) let files := children.filter Hierarchy.isFile |>.map Hierarchy.getName let dirNodes ← (dirs.mapM moduleListDir) let fileNodes ← (files.mapM moduleListFile) let attributes := match ←getCurrentName with | some name => if h.getName.isPrefixOf name then #[("class", "nav_sect"), ("data-path", moduleNameToUrl h.getName), ("open", "")] else #[("class", "nav_sect"), ("data-path", moduleNameToUrl h.getName)] | none => #[("class", "nav_sect"), ("data-path", moduleNameToUrl h.getName)] let nodes := #[{h.getName.toString}] ++ dirNodes ++ fileNodes return Html.element "details" attributes nodes def moduleList : HtmlM (Array Html) := do let hierarchy := (←getResult).hierarchy let mut list := Array.empty for (n, cs) in hierarchy.getChildren do list := list.push

{n.toString}

list := list.push $ ←moduleListDir cs list def navbar : HtmlM Html := do end Output end DocGen4