diff -r a29295dac1ca -r f92bf6674699 src/HOL/Hahn_Banach/Vector_Space.thy --- a/src/HOL/Hahn_Banach/Vector_Space.thy Mon Nov 02 11:10:28 2015 +0100 +++ b/src/HOL/Hahn_Banach/Vector_Space.thy Mon Nov 02 11:43:02 2015 +0100 @@ -11,9 +11,9 @@ subsection \Signature\ text \ - For the definition of real vector spaces a type @{typ 'a} of the - sort \{plus, minus, zero}\ is considered, on which a real - scalar multiplication \\\ is declared. + For the definition of real vector spaces a type @{typ 'a} of the sort + \{plus, minus, zero}\ is considered, on which a real scalar multiplication + \\\ is declared. \ consts @@ -23,13 +23,13 @@ subsection \Vector space laws\ text \ - A \<^emph>\vector space\ is a non-empty set \V\ of elements from - @{typ 'a} with the following vector space laws: The set \V\ is - closed under addition and scalar multiplication, addition is - associative and commutative; \- x\ is the inverse of \x\ w.~r.~t.~addition and \0\ is the neutral element of - addition. Addition and multiplication are distributive; scalar - multiplication is associative and the real number \1\ is - the neutral element of scalar multiplication. + A \<^emph>\vector space\ is a non-empty set \V\ of elements from @{typ 'a} with + the following vector space laws: The set \V\ is closed under addition and + scalar multiplication, addition is associative and commutative; \- x\ is + the inverse of \x\ wrt.\ addition and \0\ is the neutral element of + addition. Addition and multiplication are distributive; scalar + multiplication is associative and the real number \1\ is the neutral + element of scalar multiplication. \ locale vectorspace = @@ -64,7 +64,8 @@ lemma neg_closed [iff]: "x \ V \ - x \ V" by (simp add: negate_eq1) -lemma add_left_commute: "x \ V \ y \ V \ z \ V \ x + (y + z) = y + (x + z)" +lemma add_left_commute: + "x \ V \ y \ V \ z \ V \ x + (y + z) = y + (x + z)" proof - assume xyz: "x \ V" "y \ V" "z \ V" then have "x + (y + z) = (x + y) + z" @@ -77,8 +78,8 @@ lemmas add_ac = add_assoc add_commute add_left_commute -text \The existence of the zero element of a vector space - follows from the non-emptiness of carrier set.\ +text \The existence of the zero element of a vector space follows from the + non-emptiness of carrier set.\ lemma zero [iff]: "0 \ V" proof - @@ -213,7 +214,8 @@ then show "x + y = x + z" by (simp only:) qed -lemma add_right_cancel: "x \ V \ y \ V \ z \ V \ (y + x = z + x) = (y = z)" +lemma add_right_cancel: + "x \ V \ y \ V \ z \ V \ (y + x = z + x) = (y = z)" by (simp only: add_commute add_left_cancel) lemma add_assoc_cong: @@ -371,4 +373,3 @@ end end -