src/HOL/Matrix_LP/Matrix.thy
changeset 54864 a064732223ad
parent 54230 b1d955791529
child 57512 cc97b347b301
equal deleted inserted replaced
54863:82acc20ded73 54864:a064732223ad
  1268   shows
  1268   shows
  1269   "transpose_matrix (mult_matrix fmul fadd A B) = mult_matrix fmul fadd (transpose_matrix B) (transpose_matrix A)"
  1269   "transpose_matrix (mult_matrix fmul fadd A B) = mult_matrix fmul fadd (transpose_matrix B) (transpose_matrix A)"
  1270   apply (simp add: Rep_matrix_inject[THEN sym])
  1270   apply (simp add: Rep_matrix_inject[THEN sym])
  1271   apply (rule ext)+
  1271   apply (rule ext)+
  1272   using assms
  1272   using assms
  1273   apply (simp add: Rep_mult_matrix max_ac)
  1273   apply (simp add: Rep_mult_matrix ac_simps)
  1274   done
  1274   done
  1275 
  1275 
  1276 lemma column_transpose_matrix: "column_of_matrix (transpose_matrix A) n = transpose_matrix (row_of_matrix A n)"
  1276 lemma column_transpose_matrix: "column_of_matrix (transpose_matrix A) n = transpose_matrix (row_of_matrix A n)"
  1277 apply (simp add:  Rep_matrix_inject[THEN sym])
  1277 apply (simp add:  Rep_matrix_inject[THEN sym])
  1278 apply (rule ext)+
  1278 apply (rule ext)+