Documentation

Lean.Meta.Tactic.Grind.Arith.Linear.Proof

Returns a context of type RArray α containing the variables of the given structure, where α is (← getStruct).type.

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

    Similar to toContextExpr, but for the CommRing module. Recall that this module interfaces with the CommRing module and their variable contexts may not be necessarily identical. For example, for this module, the term x*y does not have an interpretation and we have a "variable" representing it, but it is interpreted in the CommRing module, and such variable does not exist there. On the other direction, suppose we have the inequality z < 0, and z does not occur in any equality or disequality. Then, the CommRing does not even "see" z, and z does not occur in its context, but it occurs in the variable context created by this module.

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

        Auxiliary monad for constructing linarith proofs.

        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.
              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

                    A linarith proof may depend on decision variables. We collect them and perform non chronological backtracking.