(* Title: HOL/Matrix/cplex/Cplex.thy ID: $Id$ Author: Steven Obua *) theory Cplex imports FloatSparseMatrix uses "Cplex_tools.ML" "CplexMatrixConverter.ML" "FloatSparseMatrixBuilder.ML" "fspmlp.ML" begin end