Documentation

Mathlib.Tactic.Linarith.SimplexAlgorithm.Datatypes

Datatypes for Simplex Algorithm implementation #

Structure for matrices over ℚ.

So far it is just a 2d-array carrying dimensions (that are supposed to match with the actual dimensions of data), but the plan is to add some Prop-data and make the structure strict and safe.

Note: we avoid using the Matrix from Mathlib.Data.Matrix because it is far more efficient to store matrix as its entries than as function between Fin-s.

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

    Table is a structure Simplex Algorithm operates on. The i-th row of mat expresses the variable basic[i] as a linear combination of variables from free.

    • basic : Array Nat

      Array containing the basic variables' indexes

    • free : Array Nat

      Array containing the free variables' indexes

    • mat : Linarith.SimplexAlgorithm.Matrix self.basic.size self.free.size

      Matrix of coefficients the basic variables expressed through the free ones.

    Instances For