src/HOL/Matrix/cplex/Cplex.thy
changeset 16784 92ff7c903585
child 16890 c4e5afaba440
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Matrix/cplex/Cplex.thy	Wed Jul 13 09:53:50 2005 +0200
@@ -0,0 +1,14 @@
+(*  Title:      HOL/Matrix/cplex/Cplex.thy
+    ID:         $Id$
+    Author:     Steven Obua
+*)
+
+theory Cplex 
+imports FloatSparseMatrix
+files "Cplex_tools.ML" "CplexMatrixConverter.ML" "FloatSparseMatrixBuilder.ML" "fspmlp.ML"
+begin
+
+end
+
+
+