diff -r b07ae33cc459 -r 202a09ba37d8 src/HOL/Matrix/SparseMatrix.thy --- a/src/HOL/Matrix/SparseMatrix.thy Mon Feb 27 10:56:36 2012 +0100 +++ b/src/HOL/Matrix/SparseMatrix.thy Mon Feb 27 11:38:56 2012 +0100 @@ -97,7 +97,7 @@ apply (auto) apply (frule sorted_spvec_cons2, simp) apply (frule sorted_spvec_cons3, simp) - apply (simp add: sparse_row_matrix_cons neg_def) + apply (simp add: sparse_row_matrix_cons) done primrec minus_spvec :: "('a::ab_group_add) spvec \ 'a spvec" @@ -273,7 +273,6 @@ apply (simp add: algebra_simps sparse_row_matrix_cons) apply (simplesubst Rep_matrix_zero_imp_mult_zero) apply (simp) - apply (intro strip) apply (rule disjI2) apply (intro strip) apply (subst nrows) @@ -284,7 +283,6 @@ apply (case_tac "k <= j") apply (rule_tac m1 = k and n1 = i and a1 = a in ssubst[OF sorted_sparse_row_vector_zero]) apply (simp_all) - apply (rule impI) apply (rule disjI2) apply (rule nrows) apply (rule order_trans[of _ 1]) @@ -297,7 +295,7 @@ apply (simp) apply (rule disjI2) apply (intro strip) - apply (simp add: sparse_row_matrix_cons neg_def) + apply (simp add: sparse_row_matrix_cons) apply (case_tac "i <= j") apply (erule sorted_sparse_row_matrix_zero) apply (simp_all) @@ -315,7 +313,6 @@ apply (auto) apply (rule_tac m=k and n = j and a = a and arr=arr in sorted_sparse_row_vector_zero) apply (simp_all) - apply (simp add: neg_def) apply (drule nrows_notzero) apply (drule nrows_helper) apply (arith) @@ -647,7 +644,7 @@ lemma disj_move_sparse_vec_mat[simplified disj_matrices_commute]: "j <= a \ sorted_spvec((a,c)#as) \ disj_matrices (move_matrix (sparse_row_vector b) (int j) i) (sparse_row_matrix as)" - apply (auto simp add: neg_def disj_matrices_def) + apply (auto simp add: disj_matrices_def) apply (drule nrows_notzero) apply (drule less_le_trans[OF _ nrows_spvec]) apply (subgoal_tac "ja = j") @@ -664,7 +661,7 @@ lemma disj_move_sparse_row_vector_twice: "j \ u \ disj_matrices (move_matrix (sparse_row_vector a) j i) (move_matrix (sparse_row_vector b) u v)" - apply (auto simp add: neg_def disj_matrices_def) + apply (auto simp add: disj_matrices_def) apply (rule nrows, rule order_trans[of _ 1], simp, drule nrows_notzero, drule less_le_trans[OF _ nrows_spvec], arith)+ done @@ -783,7 +780,7 @@ apply (simplesubst sorted_sparse_row_matrix_zero) apply auto apply (simplesubst Rep_sparse_row_vector_zero) - apply (simp_all add: neg_def) + apply simp_all done lemma sorted_spvec_minus_spmat: "sorted_spvec A \ sorted_spvec (minus_spmat A)"