Documentation
Lean
.
Meta
.
Tactic
.
Unfold
Search
return to top
source
Imports
Lean.Meta.Eqns
Lean.Meta.Tactic.Delta
Lean.Meta.Tactic.Simp.Main
Imported by
Lean
.
Meta
.
unfold
Lean
.
Meta
.
unfold
.
pre
Lean
.
Meta
.
unfoldTarget
Lean
.
Meta
.
unfoldLocalDecl
Lean
.
Meta
.
zetaDeltaTarget
Lean
.
Meta
.
zetaDeltaLocalDecl
source
def
Lean
.
Meta
.
unfold
(e :
Expr
)
(declName :
Name
)
:
MetaM
Simp.Result
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
unfold
.
pre
(unfoldThm :
Name
)
(e :
Expr
)
:
SimpM
Simp.Step
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
unfoldTarget
(mvarId :
MVarId
)
(declName :
Name
)
:
MetaM
MVarId
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
unfoldLocalDecl
(mvarId :
MVarId
)
(fvarId :
FVarId
)
(declName :
Name
)
:
MetaM
MVarId
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
zetaDeltaTarget
(mvarId :
MVarId
)
(declFVarId :
FVarId
)
:
MetaM
MVarId
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
zetaDeltaLocalDecl
(mvarId :
MVarId
)
(fvarId declFVarId :
FVarId
)
:
MetaM
MVarId
Equations
One or more equations did not get rendered due to their size.
Instances For