src/HOL/Multivariate_Analysis/Determinants.thy
changeset 56196 32b7eafc5a52
parent 53854 78afb4c4e683
child 56545 8f1e7596deb7
equal deleted inserted replaced
56195:c7dfd924a165 56196:32b7eafc5a52
   962   have "(\<chi> i. row i A) = A" by (vector row_def)
   962   have "(\<chi> i. row i A) = A" by (vector row_def)
   963   then have thd1: "det (\<chi> i. row i A) = det A"
   963   then have thd1: "det (\<chi> i. row i A) = det A"
   964     by simp
   964     by simp
   965   have thd0: "det (\<chi> i. if i = k then row k A + (\<Sum>i \<in> ?Uk. x $ i *s row i A) else row i A) = det A"
   965   have thd0: "det (\<chi> i. if i = k then row k A + (\<Sum>i \<in> ?Uk. x $ i *s row i A) else row i A) = det A"
   966     apply (rule det_row_span)
   966     apply (rule det_row_span)
   967     apply (rule span_setsum[OF fUk])
   967     apply (rule span_setsum)
   968     apply (rule ballI)
   968     apply (rule ballI)
   969     apply (rule span_mul [where 'a="real^'n", folded scalar_mult_eq_scaleR])+
   969     apply (rule span_mul [where 'a="real^'n", folded scalar_mult_eq_scaleR])+
   970     apply (rule span_superset)
   970     apply (rule span_superset)
   971     apply auto
   971     apply auto
   972     done
   972     done