src/HOL/Matrix/cplex/FloatSparseMatrix.thy
changeset 27484 dbb9981c3d18
parent 27483 7c58324cd418
child 27485 a5de2cbf548f
--- a/src/HOL/Matrix/cplex/FloatSparseMatrix.thy	Thu Jul 03 20:53:44 2008 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,10 +0,0 @@
-(*  Title:      HOL/Matrix/cplex/FloatSparseMatrix.thy
-    ID:         $Id$
-    Author:     Steven Obua
-*)
-
-theory FloatSparseMatrix
-imports "../../Real/Float" SparseMatrix
-begin
-
-end