Equations
- Lean.Elab.Tactic.isHoleRHS rhs = (rhs.isOfKind `Lean.Parser.Term.syntheticHole || rhs.isOfKind `Lean.Parser.Term.hole)
Instances For
Helper method for creating an user-defined eliminator/recursor application.
- name : Name
The short name of the alternative, used in
| foo =>
cases - info : Meta.ElimAltInfo
- mvarId : MVarId
The subgoal metavariable for the alternative.
Instances For
Equations
- Lean.Elab.Tactic.ElimApp.instInhabitedAlt = { default := { name := default, info := default, mvarId := default } }
- elimInfo : Meta.ElimInfo
Instances For
@[reducible, inline]
Equations
Instances For
def
Lean.Elab.Tactic.ElimApp.mkElimApp
(elimInfo : Meta.ElimInfo)
(targets : Array Expr)
(tag : Name)
:
Construct the an eliminator/recursor application. targets
contains the explicit and implicit targets for
the eliminator. For example, the indices of builtin recursors are considered implicit targets.
Remark: the method addImplicitTargets
may be used to compute the sequence of implicit and explicit targets
from the explicit ones.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.ElimApp.evalAlts
(elimInfo : Meta.ElimInfo)
(alts : Array Alt)
(optPreTac : Syntax)
(altStxs : Array Syntax)
(initialInfo : Info)
(numEqs numGeneralized : Nat := 0)
(toClear : Array FVarId := #[])
(toTag : Array (Ident × FVarId) := #[])
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.ElimApp.evalAlts.goWithInfo
(elimInfo : Meta.ElimInfo)
(alts : Array Alt)
(optPreTac : Syntax)
(altStxs : Array Syntax)
(numEqs numGeneralized : Nat := 0)
(toClear : Array FVarId := #[])
(toTag : Array (Ident × FVarId) := #[])
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.ElimApp.evalAlts.goWithIncremental
(elimInfo : Meta.ElimInfo)
(alts : Array Alt)
(optPreTac : Syntax)
(altStxs : Array Syntax)
(numEqs numGeneralized : Nat := 0)
(toClear : Array FVarId := #[])
(toTag : Array (Ident × FVarId) := #[])
(tacSnaps : Array (Language.SnapshotBundle TacticParsedSnapshot))
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.ElimApp.evalAlts.applyAltStx
(elimInfo : Meta.ElimInfo)
(optPreTac : Syntax)
(altStxs : Array Syntax)
(numEqs numGeneralized : Nat := 0)
(toClear : Array FVarId := #[])
(toTag : Array (Ident × FVarId) := #[])
(tacSnaps : Array (Language.SnapshotBundle TacticParsedSnapshot))
(altStxIdx : Nat)
(altStx : Syntax)
(alt : Alt)
:
Applies syntactic alternative to alternative goal.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.