src/HOL/Analysis/Finite_Cartesian_Product.thy
changeset 69272 15e9ed5b28fb
parent 69260 0a9688695a1b
child 69517 dc20f278e8f3
--- a/src/HOL/Analysis/Finite_Cartesian_Product.thy	Thu Nov 08 22:02:07 2018 +0100
+++ b/src/HOL/Analysis/Finite_Cartesian_Product.thy	Thu Nov 08 22:29:09 2018 +0100
@@ -1228,7 +1228,7 @@
 proof%unimportant -
   obtain A' where "A ** A' = mat 1" and "A' ** A = mat 1"
     using assms unfolding invertible_def by auto
-  with `k \<noteq> 0`
+  with \<open>k \<noteq> 0\<close>
   have "(k *\<^sub>R A) ** ((1/k) *\<^sub>R A') = mat 1" "((1/k) *\<^sub>R A') ** (k *\<^sub>R A) = mat 1"
     by (simp_all add: assms matrix_scalar_ac)
   thus "invertible (k *\<^sub>R A)"