src/HOL/Matrix_LP/Cplex.thy
changeset 48891 c0eafbd55de3
parent 47455 26315a545e26
child 69605 a96320074298
--- a/src/HOL/Matrix_LP/Cplex.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/src/HOL/Matrix_LP/Cplex.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -4,10 +4,13 @@
 
 theory Cplex 
 imports SparseMatrix LP ComputeFloat ComputeNumeral
-uses "Cplex_tools.ML" "CplexMatrixConverter.ML" "FloatSparseMatrixBuilder.ML"
-  "fspmlp.ML" ("matrixlp.ML")
 begin
 
+ML_file "Cplex_tools.ML"
+ML_file "CplexMatrixConverter.ML"
+ML_file "FloatSparseMatrixBuilder.ML"
+ML_file "fspmlp.ML"
+
 lemma spm_mult_le_dual_prts: 
   assumes
   "sorted_sparse_matrix A1"
@@ -61,7 +64,7 @@
   (mult_est_spmat r1 r2 (diff_spmat c1 (mult_spmat y A2)) (diff_spmat c2 (mult_spmat y A1))))"
   by (simp add: assms mult_est_spmat_def spm_mult_le_dual_prts[where A=A, simplified Let_def])
 
-use "matrixlp.ML"
+ML_file "matrixlp.ML"
 
 end