src/HOL/Matrix/cplex/MatrixLP.thy
author huffman
Tue, 01 Jul 2008 01:09:03 +0200
changeset 27406 3897988917a3
parent 23665 825bea0266db
permissions -rw-r--r--
rename compact_approx to compact_take
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
16873
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     1
(*  Title:      HOL/Matrix/cplex/MatrixLP.thy
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     2
    ID:         $Id$
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     3
    Author:     Steven Obua
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     4
*)
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     5
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     6
theory MatrixLP 
23665
825bea0266db adopted to new computing oracle and fixed bugs introduced by tuning
obua
parents: 23174
diff changeset
     7
imports Cplex 
825bea0266db adopted to new computing oracle and fixed bugs introduced by tuning
obua
parents: 23174
diff changeset
     8
uses "matrixlp.ML"
16873
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
     9
begin
9ed940a1bebb proving bounds for real linear programs
obua
parents:
diff changeset
    10
end