Documentation

Lean.Meta.Tactic.Grind.Order.Proof

Returns declName α leInst isPreorderInst

Equations
Instances For

    Returns declName α leInst ltInst lawfulOrderLtInst isLinearPreorderInst

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

      Returns declName α leInst isLinearPreorderInst

      Equations
      Instances For

        Returns declName α leInst ltInst lawfulOrderLtInst isPreorderInst ringInst ordRingInst

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

          Returns declName α leInst ltInst lawfulOrderLtInst isLinearPreorderInst ringInst ordRingInst

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

            Assume p₁ is { w := u, k := k₁, proof := p₁ } and p₂ is { w := w, k := k₂, proof := p₂ } p₁ is the proof for edge u -(k₁)→ w and p₂ the proof for edge w -(k₂)-> v. Then, this function returns a proof for edge u -(k₁+k₂) -> v.

            Remark: if the order does not support offset k₁ and k₂ are zero.

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

              Given a path u --(k)--> v justified by proof huv, construct a proof of e = True where e is a term corresponding to the edge u --(k') --> v

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

                Constructs a proof of e = True where e is a term corresponding to the edge u --(k) --> u with k non-negative

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

                  Given a path u --(k)--> v justified by proof huv, construct a proof of e = False where e is a term corresponding to the edge u --(k') --> v

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

                    Constructs a proof of e = False where e is a term corresponding to the edge u --(k) --> u and k is negative.

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

                      Returns a proof of False using u --(k)--> u with proof h where k is negative

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        def Lean.Meta.Grind.Order.mkUnsatProof (u v : Expr) (k₁ : Weight) (h₁ : Expr) (k₂ : Weight) (h₂ : Expr) :

                        Returns a proof of False using a negative cycle composed of

                        • u --(k₁)--> v with proof h₁
                        • v --(k₂)--> u with proof h₂
                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          Equations
                          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