Documentation

Lean.Meta.Tactic.Grind.Arith.Linear.Util

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

    We don't want to keep carrying the StructId around.

    Equations
    Instances For
      @[reducible, inline]
      abbrev Lean.Meta.Grind.Arith.Linear.LinearM.run {α : Type} (structId : Nat) (x : LinearM α) :
      Equations
      Instances For
        @[reducible, inline]
        Equations
        Instances For
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            Equations
            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
                    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
                        @[inline]
                        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
                                    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

                                              Tries to evaluate the polynomial p using the partial model/assignment built so far. The result is none if the polynomial contains variables that have not been assigned.

                                              Equations
                                              Instances For

                                                Returns .true if c is satisfied by the current partial model, .undef if c contains unassigned variables, and .false otherwise.

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

                                                    Resets the assignment of any variable bigger or equal to x.

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

                                                      Returns true if the linarith state is inconsistent.

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

                                                        Returns true if x has been eliminated using an equality constraint.

                                                        Equations
                                                        Instances For

                                                          Adds y as an occurrence of x. That is, x occurs in lowers[y], uppers[y], or diseqs[y].

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

                                                            Given p a polynomial being inserted into lowers, uppers, or diseqs, get its leading variable y, and adds y as an occurrence for the remaining variables in p.

                                                            Equations
                                                            Instances For

                                                              Given a polynomial p, returns some (x, k, c) if p contains the monomial k*x, and x has been eliminated using the equality c.

                                                              Equations
                                                              Instances For

                                                                Selects the variable in the given linear polynomial whose coefficient has the smallest absolute value.

                                                                Equations
                                                                Instances For
                                                                  Equations
                                                                  Instances For