Documentation
Lean
.
Compiler
.
LCNF
.
AuxDeclCache
Search
return to top
source
Imports
Lean.Compiler.LCNF.CompilerM
Lean.Compiler.LCNF.DeclHash
Lean.Compiler.LCNF.Internalize
Imported by
Lean
.
Compiler
.
LCNF
.
AuxDeclCache
Lean
.
Compiler
.
LCNF
.
auxDeclCacheExt
Lean
.
Compiler
.
LCNF
.
CacheAuxDeclResult
Lean
.
Compiler
.
LCNF
.
cacheAuxDecl
source
@[reducible, inline]
abbrev
Lean
.
Compiler
.
LCNF
.
AuxDeclCache
:
Type
Equations
Lean.Compiler.LCNF.AuxDeclCache
=
Lean.PHashMap
Lean.Compiler.LCNF.Decl
Lean.Name
Instances For
source
opaque
Lean
.
Compiler
.
LCNF
.
auxDeclCacheExt
:
EnvExtension
AuxDeclCache
source
inductive
Lean
.
Compiler
.
LCNF
.
CacheAuxDeclResult
:
Type
new :
CacheAuxDeclResult
alreadyCached
(declName :
Name
)
:
CacheAuxDeclResult
Instances For
source
def
Lean
.
Compiler
.
LCNF
.
cacheAuxDecl
(decl :
Decl
)
:
CompilerM
CacheAuxDeclResult
Equations
One or more equations did not get rendered due to their size.
Instances For