src/HOL/Matrix/cplex/MatrixLP.thy
author wenzelm
Thu, 28 Feb 2008 00:11:28 +0100
changeset 26173 5cac519abe4e
parent 23665 825bea0266db
permissions -rw-r--r--
renamed ListSpace to ListVector;

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

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