Documentation

Mathlib.Tactic.Linarith.Oracle.SimplexAlgorithm.Gauss

Gaussian Elimination algorithm #

The first step of Linarith.SimplexAlgorithm.findPositiveVector is finding initial feasible solution which is done by standard Gaussian Elimination algorithm implemented in this file.

@[reducible, inline]
abbrev Linarith.SimplexAlgorithm.Gauss.GaussM (n : Nat) (m : Nat) (matType : NatNatType) (α : Type) :

The monad for the Gaussian Elimination algorithm.

Equations
Instances For

    Finds the first row starting from the rowStart with nonzero element in the column col.

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

      Implementation of getTableau in GaussM monad.

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

        Given matrix A, solves the linear equation A x = 0 and returns the solution as a tableau where some variables are free and others (basic) variable are expressed as linear combinations of the free ones.

        Equations
        Instances For