src/HOL/Matrix/MatrixLP.thy
author nipkow
Fri, 18 Feb 2005 15:20:27 +0100
changeset 15537 5538d3244b4d
parent 15178 5f621aa35c25
permissions -rw-r--r--
continued eliminating sumr
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
15178
5f621aa35c25 Matrix theory, linear programming
obua
parents:
diff changeset
     1
theory MatrixLP = Float + SparseMatrix:
5f621aa35c25 Matrix theory, linear programming
obua
parents:
diff changeset
     2
5f621aa35c25 Matrix theory, linear programming
obua
parents:
diff changeset
     3
end
5f621aa35c25 Matrix theory, linear programming
obua
parents:
diff changeset
     4