src/HOL/Matrix/cplex/MatrixLP.thy
author obua
Fri, 17 Aug 2007 09:20:45 +0200
changeset 24302 3045683749af
parent 23665 825bea0266db
permissions -rw-r--r--
tuned

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

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