Documentation
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
Basic
Search
return to top
source
Imports
Lean.Meta
Std.Tactic.Do.Syntax
Lean.Elab.Tactic.Do.ProofMode.MGoal
Imported by
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
MStartResult
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
mStart
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
mStartMVar
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
elabMStart
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
elabMStop
source
structure
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
MStartResult
:
Type
goal :
MGoal
proof? :
Option
Expr
Instances For
source
def
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
mStart
(
goal
:
Expr
)
:
MetaM
MStartResult
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
mStartMVar
(
mvar
:
MVarId
)
:
MetaM
(
MVarId
×
MGoal
)
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
elabMStart
:
Tactic
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Elab
.
Tactic
.
Do
.
ProofMode
.
elabMStop
:
Tactic
Equations
One or more equations did not get rendered due to their size.
Instances For