src/HOL/Matrix/SparseMatrix.thy
changeset 24124 4399175e3014
parent 23477 f4b83f03cac9
child 25303 0699e20feabd
--- a/src/HOL/Matrix/SparseMatrix.thy	Wed Aug 01 21:10:36 2007 +0200
+++ b/src/HOL/Matrix/SparseMatrix.thy	Thu Aug 02 12:06:27 2007 +0200
@@ -600,7 +600,7 @@
   disj_matrices :: "('a::zero) matrix \<Rightarrow> 'a matrix \<Rightarrow> bool"
   "disj_matrices A B == (! j i. (Rep_matrix A j i \<noteq> 0) \<longrightarrow> (Rep_matrix B j i = 0)) & (! j i. (Rep_matrix B j i \<noteq> 0) \<longrightarrow> (Rep_matrix A j i = 0))"  
 
-ML {* simp_depth_limit := 6 *}
+declare [[simp_depth_limit = 6]]
 
 lemma disj_matrices_contr1: "disj_matrices A B \<Longrightarrow> Rep_matrix A j i \<noteq> 0 \<Longrightarrow> Rep_matrix B j i = 0"
    by (simp add: disj_matrices_def)
@@ -777,7 +777,7 @@
   apply (simp add: sorted_spvec_cons1 le_spvec_iff_sparse_row_le)
   done
 
-ML {* simp_depth_limit := 999 *}
+declare [[simp_depth_limit = 999]]
 
 consts 
    abs_spmat :: "('a::lordered_ring) spmat \<Rightarrow> 'a spmat"