20 lines
445 B
Plaintext
20 lines
445 B
Plaintext
/-
|
|
Copyright (c) 2022 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.Base
|
|
import DocGen4.Process.NameInfo
|
|
|
|
namespace DocGen4.Process
|
|
|
|
open Lean Meta
|
|
|
|
def AxiomInfo.ofAxiomVal (v : AxiomVal) : MetaM AxiomInfo := do
|
|
let info ← Info.ofConstantVal v.toConstantVal
|
|
pure <| AxiomInfo.mk info v.isUnsafe
|
|
|
|
end DocGen4.Process
|