bookshelf-doc/DocGen4/Output/ToJson.lean

127 lines
4.5 KiB
Plaintext
Raw Normal View History

import Lean
import DocGen4.Process
import DocGen4.Output.Base
2023-08-06 13:36:43 +00:00
import DocGen4.Output.Module
import Lean.Data.RBMap
namespace DocGen4.Output
open Lean
2023-08-06 13:36:43 +00:00
structure JsonDeclarationInfo where
name : String
kind : String
doc : String
docLink : String
sourceLink : String
2023-08-06 13:36:43 +00:00
line : Nat
deriving FromJson, ToJson
2023-08-06 13:36:43 +00:00
structure JsonDeclaration where
info : JsonDeclarationInfo
header : String
deriving FromJson, ToJson
structure JsonInstance where
name : String
className : String
2022-07-23 13:40:08 +00:00
typeNames : Array String
deriving FromJson, ToJson
structure JsonModule where
name : String
declarations : List JsonDeclaration
instances : Array JsonInstance
imports : Array String
deriving FromJson, ToJson
2023-08-06 13:36:43 +00:00
structure JsonHeaderIndex where
headers : List (String × String) := []
2022-07-23 18:40:08 +00:00
structure JsonIndex where
2023-08-06 13:36:43 +00:00
declarations : List (String × JsonDeclarationInfo) := []
instances : HashMap String (RBTree String Ord.compare) := .empty
2022-07-23 18:40:08 +00:00
importedBy : HashMap String (Array String) := .empty
modules : List (String × String) := []
instancesFor : HashMap String (RBTree String Ord.compare) := .empty
2022-07-23 18:40:08 +00:00
2023-08-06 13:36:43 +00:00
instance : ToJson JsonHeaderIndex where
toJson idx := Json.mkObj <| idx.headers.map (fun (k, v) => (k, toJson v))
2022-07-23 18:40:08 +00:00
instance : ToJson JsonIndex where
toJson idx := Id.run do
2023-01-01 18:51:01 +00:00
let jsonDecls := Json.mkObj <| idx.declarations.map (fun (k, v) => (k, toJson v))
let jsonInstances := Json.mkObj <| idx.instances.toList.map (fun (k, v) => (k, toJson v.toArray))
2023-01-01 18:51:01 +00:00
let jsonImportedBy := Json.mkObj <| idx.importedBy.toList.map (fun (k, v) => (k, toJson v))
let jsonModules := Json.mkObj <| idx.modules.map (fun (k, v) => (k, toJson v))
let jsonInstancesFor := Json.mkObj <| idx.instancesFor.toList.map (fun (k, v) => (k, toJson v.toArray))
2022-07-23 18:40:08 +00:00
let finalJson := Json.mkObj [
("declarations", jsonDecls),
("instances", jsonInstances),
("importedBy", jsonImportedBy),
("modules", jsonModules),
("instancesFor", jsonInstancesFor)
]
2023-01-01 18:51:01 +00:00
return finalJson
2022-07-23 18:40:08 +00:00
2023-08-06 13:36:43 +00:00
def JsonHeaderIndex.addModule (index : JsonHeaderIndex) (module : JsonModule) : JsonHeaderIndex :=
let merge idx decl := { idx with headers := (decl.info.name, decl.header) :: idx.headers }
module.declarations.foldl merge index
2022-07-23 18:40:08 +00:00
def JsonIndex.addModule (index : JsonIndex) (module : JsonModule) : BaseHtmlM JsonIndex := do
let mut index := index
2023-01-01 18:51:01 +00:00
let newModule := (module.name, ← moduleNameToLink (String.toName module.name))
2023-08-06 13:36:43 +00:00
let newDecls := module.declarations.map (fun d => (d.info.name, d.info))
2022-07-23 18:40:08 +00:00
index := { index with
modules := newModule :: index.modules
declarations := newDecls ++ index.declarations
}
-- TODO: In theory one could sort instances and imports by name and batch the writes
for inst in module.instances do
let mut insts := index.instances.findD inst.className {}
insts := insts.insert inst.name
2022-07-23 18:40:08 +00:00
index := { index with instances := index.instances.insert inst.className insts }
for typeName in inst.typeNames do
let mut instsFor := index.instancesFor.findD typeName {}
instsFor := instsFor.insert inst.name
2022-07-23 18:40:08 +00:00
index := { index with instancesFor := index.instancesFor.insert typeName instsFor }
for imp in module.imports do
let mut impBy := index.importedBy.findD imp #[]
impBy := impBy.push module.name
index := { index with importedBy := index.importedBy.insert imp impBy }
2023-01-01 18:51:01 +00:00
return index
2022-07-23 18:40:08 +00:00
def DocInfo.toJson (module : Name) (info : Process.DocInfo) : HtmlM JsonDeclaration := do
let name := info.getName.toString
let kind := info.getKind
let doc := info.getDocString.getD ""
let docLink ← declNameToLink info.getName
let sourceLink ← getSourceUrl module info.getDeclarationRange
2023-08-06 13:36:43 +00:00
let line := info.getDeclarationRange.pos.line
let header := (← docInfoHeader info).toString
let info := { name, kind, doc, docLink, sourceLink, line }
return { info, header }
def Process.Module.toJson (module : Process.Module) : HtmlM Json := do
let mut jsonDecls := []
let mut instances := #[]
2023-02-16 18:51:35 +00:00
let declInfo := Process.filterDocInfo module.members
for decl in declInfo do
2023-01-01 18:51:01 +00:00
jsonDecls := (← DocInfo.toJson module.name decl) :: jsonDecls
if let .instanceInfo i := decl then
2022-07-23 13:40:08 +00:00
instances := instances.push {
name := i.name.toString,
className := i.className.toString
typeNames := i.typeNames.map Name.toString
}
let jsonMod : JsonModule := {
name := module.name.toString,
declarations := jsonDecls,
2022-07-23 13:40:08 +00:00
instances,
imports := module.imports.map Name.toString
}
2023-01-01 18:51:01 +00:00
return ToJson.toJson jsonMod
end DocGen4.Output