Documentation
Lean
.
Elab
.
Tactic
.
Delta
Search
return to top
source
Imports
Lean.Elab.Tactic.Basic
Lean.Elab.Tactic.Location
Lean.Meta.Tactic.Delta
Imported by
Lean
.
Elab
.
Tactic
.
deltaLocalDecl
Lean
.
Elab
.
Tactic
.
deltaTarget
Lean
.
Elab
.
Tactic
.
evalDelta
source
def
Lean
.
Elab
.
Tactic
.
deltaLocalDecl
(declNames :
Array
Name
)
(fvarId :
FVarId
)
:
TacticM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Tactic
.
deltaTarget
(declNames :
Array
Name
)
:
TacticM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Tactic
.
evalDelta
:
Tactic
"delta " ident+ (location)?
Equations
One or more equations did not get rendered due to their size.
Instances For