Documentation

Lean.Elab.Tactic.Basic

Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
  • Declaration name of the executing elaborator, used by mkTacticInfo to persist it in the info tree

    elaborator : Lean.Name
  • If true, enable "error recovery" in some tactics. For example, cases tactic admits unsolved alternatives when recover == true. The combinator withoutRecover disables "error recovery" while executing . This is useful for tactics such as first | ... | ....

    recover : Bool
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations

Execute x with error recovery disabled

Equations
Equations
  • Lean.Elab.Tactic.instOrElseTacticM = { orElse := Lean.Elab.Tactic.orElse }
@[inline]
Equations
  • One or more equations did not get rendered due to their size.

Adapt a syntax transformation to a regular tactic evaluator.

Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations

Execute x using the main goal local context and instances

Equations

Evaluate tac at mvarId, and return the list of resulting subgoals.

Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.

Close main goal using the given expression. If checkUnassigned == true, then val must not contain unassinged metavariables.

Equations
  • One or more equations did not get rendered due to their size.
@[inline]
Equations
  • One or more equations did not get rendered due to their size.
@[inline]
Equations
  • One or more equations did not get rendered due to their size.
Equations

Use parentTag to tag untagged goals at newGoals. If there are multiple new untagged goals, they are named using ._ where idx > 0. If there is only one new untagged goal, then we just use parentTag

Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.Tactic.withCaseRef {m : TypeType} {α : Type} [inst : Monad m] [inst : Lean.MonadRef m] (arrow : Lean.Syntax) (body : Lean.Syntax) (x : m α) :
m α

Use position of => $body for error messages. If there is a line break before body, the message will be displayed on => only, but the "full range" for the info view will still include body.

Equations