src/HOL/Vector_Spaces.thy
changeset 69593 3dda49e08b9d
parent 69064 5840724b1d71
child 69712 dc85b5b3a532
--- a/src/HOL/Vector_Spaces.thy	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/HOL/Vector_Spaces.thy	Fri Jan 04 23:22:53 2019 +0100
@@ -826,7 +826,7 @@
   by (auto simp: that construct_in_span in_span_in_range_construct)
 
 lemma linear_independent_extend_subspace:
-  \<comment> \<open>legacy: use @{term construct} instead\<close>
+  \<comment> \<open>legacy: use \<^term>\<open>construct\<close> instead\<close>
   assumes "vs1.independent B"
   shows "\<exists>g. linear s1 s2 g \<and> (\<forall>x\<in>B. g x = f x) \<and> range g = vs2.span (f`B)"
   by (rule exI[where x="construct B f"])