Documentation

Lean.Meta.Tactic.LinearArith.Solver

Instances For
    Equations
    @[reducible, inline]
    Equations
    • a.size = a.val.size
    Instances For
      @[reducible, inline]
      Equations
      • a.get? x = if h : x.id < a.size then some a.val[x.id] else none
      Instances For
        @[reducible, inline]
        Equations
        • a.push v = { val := a.val.push v }
        Instances For
          @[reducible, inline]
          Equations
          • a.take newSize = { val := a.val.take newSize }
          Instances For
            Instances For
              @[reducible, inline]
              Equations
              • e.size = e.val.size
              Instances For
                @[reducible, inline]
                Equations
                • e.getMaxVarCoeff = e.val.back!.fst
                Instances For
                  @[reducible, inline]
                  Equations
                  • e.getMaxVar = e.val.back!.snd
                  Instances For
                    @[reducible, inline]
                    abbrev Lean.Meta.Linear.Poly.get (e : Poly) (i : Fin e.size) :
                    Equations
                    • e.get i = e.val[i]
                    Instances For
                      Equations
                      Instances For
                        Equations
                        Instances For
                          @[irreducible]
                          def Lean.Meta.Linear.Poly.add.go (e₁ e₂ : Poly) (i₁ i₂ : Nat) (r : Array (Int × Var)) :
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            def Lean.Meta.Linear.Poly.combine (d₁ : Int) (e₁ : Poly) (d₂ : Int) (e₂ : Poly) :
                            Equations
                            Instances For
                              @[irreducible]
                              def Lean.Meta.Linear.Poly.combine.go (d₁ : Int) (e₁ : Poly) (d₂ : Int) (e₂ : Poly) (i₁ i₂ : Nat) (r : Array (Int × Var)) :
                              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
                                  Instances For
                                    Instances For
                                      Equations
                                      Instances For
                                        @[reducible, inline]
                                        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
                                                Instances For
                                                  Instances For
                                                    Instances For
                                                      Equations
                                                      @[reducible, inline]
                                                      Equations
                                                      • s.getNumVars = s.lowers.size
                                                      Instances For
                                                        @[reducible, inline]
                                                        Equations
                                                        • s.currVar = s.assignment.size
                                                        Instances For
                                                          @[reducible, inline]
                                                          Equations
                                                          Instances For
                                                            @[reducible, inline]
                                                            Equations
                                                            Instances For
                                                              @[reducible, inline]
                                                              Equations
                                                              • s.assignCurr v = { lowers := s.lowers, uppers := s.uppers, int := s.int, assignment := s.assignment.push v }
                                                              Instances For
                                                                def Lean.Meta.Linear.pickAssignment? (lower : Std.Internal.Rat) (lowerIsStrict : Bool) (upper : Std.Internal.Rat) (upperIsStrict : Bool) :
                                                                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
                                                                    Instances For