Documentation
Aesop
.
Index
.
DiscrTreeConfig
Search
return to top
source
Imports
Init
Lean
Imported by
Aesop
.
indexConfig
Aesop
.
mkDiscrTreePath
Aesop
.
getUnify
Aesop
.
getMatch
source
def
Aesop
.
indexConfig
:
Lean.Meta.ConfigWithKey
The configuration used by all Aesop indices.
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Aesop
.
mkDiscrTreePath
(e :
Lean.Expr
)
:
Lean.MetaM
(
Array
Lean.Meta.DiscrTree.Key
)
Equations
Aesop.mkDiscrTreePath
e
=
Lean.Meta.withConfigWithKey
Aesop.indexConfig
(
Lean.Meta.DiscrTree.mkPath
e
)
Instances For
source
def
Aesop
.
getUnify
{α :
Type
}
(t :
Lean.Meta.DiscrTree
α
)
(e :
Lean.Expr
)
:
Lean.MetaM
(
Array
α
)
Equations
Aesop.getUnify
t
e
=
Lean.Meta.withConfigWithKey
Aesop.indexConfig
(
t
.
getUnify
e
)
Instances For
source
def
Aesop
.
getMatch
{α :
Type
}
(t :
Lean.Meta.DiscrTree
α
)
(e :
Lean.Expr
)
:
Lean.MetaM
(
Array
α
)
Equations
Aesop.getMatch
t
e
=
Lean.Meta.withConfigWithKey
Aesop.indexConfig
(
t
.
getMatch
e
)
Instances For