2023-05-11 13:27:25 +00:00
|
|
|
|
/-
|
|
|
|
|
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.Process
|
|
|
|
|
import Lean.Data.HashMap
|
|
|
|
|
|
|
|
|
|
namespace DocGen4
|
|
|
|
|
|
|
|
|
|
open Lean System IO
|
2023-11-08 01:36:00 +00:00
|
|
|
|
|
|
|
|
|
def envOfImports (imports : Array Name) : IO Environment := do
|
2023-05-11 13:27:25 +00:00
|
|
|
|
importModules (imports.map (Import.mk · false)) Options.empty
|
|
|
|
|
|
2023-11-08 01:36:00 +00:00
|
|
|
|
def loadInit (imports : Array Name) : IO Hierarchy := do
|
2023-05-11 13:27:25 +00:00
|
|
|
|
let env ← envOfImports imports
|
|
|
|
|
pure <| Hierarchy.fromArray env.header.moduleNames
|
|
|
|
|
|
|
|
|
|
/--
|
|
|
|
|
Load a list of modules from the current Lean search path into an `Environment`
|
|
|
|
|
to process for documentation.
|
|
|
|
|
-/
|
|
|
|
|
def load (task : Process.AnalyzeTask) : IO (Process.AnalyzerResult × Hierarchy) := do
|
2023-11-08 01:36:00 +00:00
|
|
|
|
initSearchPath (← findSysroot)
|
2023-05-11 13:27:25 +00:00
|
|
|
|
let env ← envOfImports task.getLoad
|
|
|
|
|
let config := {
|
|
|
|
|
-- TODO: parameterize maxHeartbeats
|
|
|
|
|
maxHeartbeats := 100000000,
|
|
|
|
|
options := ⟨[(`pp.tagAppFns, true)]⟩,
|
|
|
|
|
-- TODO: Figure out whether this could cause some bugs
|
|
|
|
|
fileName := default,
|
|
|
|
|
fileMap := default,
|
|
|
|
|
}
|
|
|
|
|
|
|
|
|
|
Prod.fst <$> Meta.MetaM.toIO (Process.process task) config { env := env } {} {}
|
|
|
|
|
|
|
|
|
|
def loadCore : IO (Process.AnalyzerResult × Hierarchy) := do
|
2023-11-08 01:36:00 +00:00
|
|
|
|
load <| .loadAll #[`Init, `Lean, `Lake]
|
2023-05-11 13:27:25 +00:00
|
|
|
|
|
|
|
|
|
end DocGen4
|