diff -r 24096e89c131 -r 6d46ad54a2ab src/HOL/Multivariate_Analysis/Fashoda.thy --- a/src/HOL/Multivariate_Analysis/Fashoda.thy Sun Sep 21 16:56:06 2014 +0200 +++ b/src/HOL/Multivariate_Analysis/Fashoda.thy Sun Sep 21 16:56:11 2014 +0200 @@ -146,7 +146,7 @@ using UNIV_2 by auto have 1: "box (- 1) (1::real^2) \ {}" unfolding interval_eq_empty_cart by auto - have 2: "continuous_on (cbox -1 1) (negatex \ sqprojection \ ?F)" + have 2: "continuous_on (cbox (- 1) 1) (negatex \ sqprojection \ ?F)" apply (intro continuous_intros continuous_on_component) unfolding * apply (rule assms)+ @@ -179,7 +179,7 @@ proof - case goal1 then obtain y :: "real^2" where y: - "y \ cbox -1 1" + "y \ cbox (- 1) 1" "x = (negatex \ sqprojection \ (\w. (f \ (\x. x $ 1)) w - (g \ (\x. x $ 2)) w)) y" unfolding image_iff .. have "?F y \ 0" @@ -208,9 +208,9 @@ qed qed obtain x :: "real^2" where x: - "x \ cbox -1 1" + "x \ cbox (- 1) 1" "(negatex \ sqprojection \ (\w. (f \ (\x. x $ 1)) w - (g \ (\x. x $ 2)) w)) x = x" - apply (rule brouwer_weak[of "cbox -1 (1::real^2)" "negatex \ sqprojection \ ?F"]) + apply (rule brouwer_weak[of "cbox (- 1) (1::real^2)" "negatex \ sqprojection \ ?F"]) apply (rule compact_cbox convex_box)+ unfolding interior_cbox apply (rule 1 2 3)+ @@ -362,7 +362,7 @@ unfolding iscale_def by auto have "\s\{- 1..1}. \t\{- 1..1}. (f \ iscale) s = (g \ iscale) t" proof (rule fashoda_unit) - show "(f \ iscale) ` {- 1..1} \ cbox -1 1" "(g \ iscale) ` {- 1..1} \ cbox -1 1" + show "(f \ iscale) ` {- 1..1} \ cbox (- 1) 1" "(g \ iscale) ` {- 1..1} \ cbox (- 1) 1" using isc and assms(3-4) by (auto simp add: image_comp [symmetric]) have *: "continuous_on {- 1..1} iscale" unfolding iscale_def by (rule continuous_intros)+ @@ -506,7 +506,7 @@ "y \ {0..1}" "x = (interval_bij (a, b) (- 1, 1) \ f) y" unfolding image_iff .. - show "x \ cbox -1 1" + show "x \ cbox (- 1) 1" unfolding y o_def apply (rule in_interval_interval_bij) using y(1) @@ -520,7 +520,7 @@ "y \ {0..1}" "x = (interval_bij (a, b) (- 1, 1) \ g) y" unfolding image_iff .. - show "x \ cbox -1 1" + show "x \ cbox (- 1) 1" unfolding y o_def apply (rule in_interval_interval_bij) using y(1)