Documentation

Lean.Elab.PreDefinition.WF.Eqns

Equations

Simplify match-expressions when trying to prove equation theorems for a recursive declaration defined using well-founded recursion. It is similar to simpMatch?, but is also tries to fold WellFounded.fix applications occurring in discriminants. See comment at tryToFoldWellFoundedFix.

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.
def Lean.Elab.WF.registerEqnsInfo (preDefs : Array Lean.Elab.PreDefinition) (declNameNonRec : Lean.Name) (fixedPrefixSize : Nat) :
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.