fixed (?) LaTeX presentation
authorpaulson <lp15@cam.ac.uk>
Mon, 02 Jul 2018 16:20:03 +0100
changeset 68571 2a6e258bfd66
parent 68570 aa48b37092df
child 68574 0307cdca6462
child 68575 d40d03487f64
fixed (?) LaTeX presentation
src/HOL/Algebra/Embedded_Algebras.thy
--- a/src/HOL/Algebra/Embedded_Algebras.thy	Mon Jul 02 15:43:22 2018 +0100
+++ b/src/HOL/Algebra/Embedded_Algebras.thy	Mon Jul 02 16:20:03 2018 +0100
@@ -122,7 +122,7 @@
 qed
 
 
-subsection \<open>Some Basic Properties of Linear_Ind\<close>
+subsection \<open>Some Basic Properties of Linear Independence\<close>
 
 lemma independent_in_carrier: "independent K Us \<Longrightarrow> set Us \<subseteq> carrier R"
   by (induct Us rule: independent.induct) (simp_all)
@@ -362,7 +362,7 @@
   using Span_eq_combine_set_length_version[OF assms] by blast
 
 
-subsection \<open>Span as the minimal subgroup that contains K <#> (set Us)\<close>
+subsection \<open>Span as the minimal subgroup that contains @{term"K <#> (set Us)"}\<close>
 
 text \<open>Now we show the link between Span and Group.generate\<close>