src/HOL/Analysis/Finite_Cartesian_Product.thy
changeset 69272 15e9ed5b28fb
parent 69260 0a9688695a1b
child 69517 dc20f278e8f3
equal deleted inserted replaced
69271:4cb70e7e36b9 69272:15e9ed5b28fb
  1226   assumes "k \<noteq> 0" and "invertible A"
  1226   assumes "k \<noteq> 0" and "invertible A"
  1227   shows "invertible (k *\<^sub>R A)"
  1227   shows "invertible (k *\<^sub>R A)"
  1228 proof%unimportant -
  1228 proof%unimportant -
  1229   obtain A' where "A ** A' = mat 1" and "A' ** A = mat 1"
  1229   obtain A' where "A ** A' = mat 1" and "A' ** A = mat 1"
  1230     using assms unfolding invertible_def by auto
  1230     using assms unfolding invertible_def by auto
  1231   with `k \<noteq> 0`
  1231   with \<open>k \<noteq> 0\<close>
  1232   have "(k *\<^sub>R A) ** ((1/k) *\<^sub>R A') = mat 1" "((1/k) *\<^sub>R A') ** (k *\<^sub>R A) = mat 1"
  1232   have "(k *\<^sub>R A) ** ((1/k) *\<^sub>R A') = mat 1" "((1/k) *\<^sub>R A') ** (k *\<^sub>R A) = mat 1"
  1233     by (simp_all add: assms matrix_scalar_ac)
  1233     by (simp_all add: assms matrix_scalar_ac)
  1234   thus "invertible (k *\<^sub>R A)"
  1234   thus "invertible (k *\<^sub>R A)"
  1235     unfolding invertible_def by auto
  1235     unfolding invertible_def by auto
  1236 qed
  1236 qed