Documentation

Lean.Meta.Tactic.ElimInfo

structure Lean.Meta.ElimAltInfo:
Type
Equations
structure Lean.Meta.ElimInfo:
Type
Equations
Equations
  • One or more equations did not get rendered due to their size.

Eliminators/recursors may have implicit targets. For builtin recursors, all indices are implicit targets. Given an eliminator and the sequence of explicit targets, this methods returns a new sequence containing implicit and explicit targets.

Equations
  • One or more equations did not get rendered due to their size.
partial def Lean.Meta.addImplicitTargets.collect (elimInfo : Lean.Meta.ElimInfo) (targets : Array Lean.Expr) (type : Lean.Expr) (argIdx : Nat) (targetIdx : Nat) (targets' : Array Lean.Expr) :
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.