src/HOL/Matrix_LP/Matrix.thy
changeset 49834 b27bbb021df1
parent 47455 26315a545e26
child 50027 7747a9f4c358
--- a/src/HOL/Matrix_LP/Matrix.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Matrix_LP/Matrix.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -13,7 +13,7 @@
 
 definition "matrix = {(f::(nat \<Rightarrow> nat \<Rightarrow> 'a::zero)). finite (nonzero_positions f)}"
 
-typedef (open) 'a matrix = "matrix :: (nat \<Rightarrow> nat \<Rightarrow> 'a::zero) set"
+typedef 'a matrix = "matrix :: (nat \<Rightarrow> nat \<Rightarrow> 'a::zero) set"
   unfolding matrix_def
 proof
   show "(\<lambda>j i. 0) \<in> {(f::(nat \<Rightarrow> nat \<Rightarrow> 'a::zero)). finite (nonzero_positions f)}"