src/HOL/Matrix/cplex/MatrixLP.thy
author haftmann
Thu, 29 May 2008 13:27:13 +0200
changeset 27014 a5f53d9d2b60
parent 23665 825bea0266db
permissions -rw-r--r--
yet another attempt to circumvent printmode problems

(*  Title:      HOL/Matrix/cplex/MatrixLP.thy
    ID:         $Id$
    Author:     Steven Obua
*)

theory MatrixLP 
imports Cplex 
uses "matrixlp.ML"
begin
end