Documentation
Lean
.
Elab
.
DocString
.
Builtin
.
Scopes
Search
return to top
source
Imports
Lean.Elab.DocString
Lean.Elab.DocString.Builtin.Parsing
Imported by
Lean
.
Doc
.
DocScope
Lean
.
Doc
.
instFromDocArgDocScope
source
inductive
Lean
.
Doc
.
DocScope
:
Type
local :
DocScope
import
(
mods
:
Array
Name
)
:
DocScope
Instances For
source
instance
Lean
.
Doc
.
instFromDocArgDocScope
:
FromDocArg
DocScope
Equations
Lean.Doc.instFromDocArgDocScope
=
{
fromDocArg
:=
fun (
v
:
Lean.Doc.DocArg
) =>
Lean.Doc.instFromDocArgDocScope._private_1
v
}