src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy
changeset 42814 5af15f1e2ef6
parent 40786 0a54cfc9add3
child 43995 c479836d9048
--- a/src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy	Sun May 15 17:06:35 2011 +0200
+++ b/src/HOL/Multivariate_Analysis/Cartesian_Euclidean_Space.thy	Sun May 15 17:45:53 2011 +0200
@@ -108,7 +108,7 @@
  in
   Attrib.thms >> (fn ths => K (SIMPLE_METHOD' (vector_arith_tac ths)))
  end
-*} "Lifts trivial vector statements to real arith statements"
+*} "lift trivial vector statements to real arith statements"
 
 lemma vec_0[simp]: "vec 0 = 0" by (vector vector_zero_def)
 lemma vec_1[simp]: "vec 1 = 1" by (vector vector_one_def)