Documentation

Lean.Elab.PreDefinition.WF.Eqns

Instances For
    Equations
    • Lean.Elab.WF.instInhabitedEqnInfo = { default := { toEqnInfoCore := default, declNames := default, declNameNonRec := default, fixedPrefixSize := default, argsPacker := default } }

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