bookshelf-doc/DocGen4/Process/AxiomInfo.lean

23 lines
469 B
Plaintext
Raw Normal View History

/-
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
return {
2022-07-23 11:37:17 +00:00
toInfo := info,
isUnsafe := v.isUnsafe
}
end DocGen4.Process