Documentation

Lean.Meta.Tactic.Grind.Order.Types

Solver for preorders, partial orders, linear orders, and support for offsets.

@[reducible, inline]
Equations
Instances For

    A constraint of the form uv + k (u < v + k if strict := true) Remark: If the order does not support offsets, then k is zero. h? := some h if the Lean expression is not definitionally equal to the constraint, but provably equal with proof h.

    Instances For
      Instances For

        Auxiliary structure used for proof extraction.

        Instances For

          Auxiliary inductive type for representing constraints and equalities that should be propagated to core. Recall that we cannot compute proofs until the short-distance data-structures have been fully updated when a new edge is inserted. Thus, we store the information to be propagated into a list. See field propagate in State.

          Instances For

            State for each order structure processed by this module. Each type must at least implement the instance Std.IsPreorder.

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

                State for all order types detected by grind.

                Instances For
                  Equations
                  Instances For