src/HOL/Matrix/SparseMatrix.thy
changeset 16417 9bc16273c2d4
parent 16041 5a8736668ced
child 16487 2060ebae96f9
--- a/src/HOL/Matrix/SparseMatrix.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Matrix/SparseMatrix.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -1,4 +1,4 @@
-theory SparseMatrix = Matrix:
+theory SparseMatrix imports Matrix begin
 
 types 
   'a spvec = "(nat * 'a) list"