diff -r ad6d4a14adb5 -r f03a01a18c6e src/HOL/Analysis/Change_Of_Vars.thy --- a/src/HOL/Analysis/Change_Of_Vars.thy Fri Apr 12 19:48:29 2019 +0200 +++ b/src/HOL/Analysis/Change_Of_Vars.thy Fri Apr 12 22:09:25 2019 +0200 @@ -424,10 +424,10 @@ subsection\\F_sigma\ and \G_delta\ sets.\(*FIX ME mv *) (*https://en.wikipedia.org/wiki/F\_set*) -inductive%important fsigma :: "'a::topological_space set \ bool" where +inductive\<^marker>\tag important\ fsigma :: "'a::topological_space set \ bool" where "(\n::nat. closed (F n)) \ fsigma (\(F ` UNIV))" -inductive%important gdelta :: "'a::topological_space set \ bool" where +inductive\<^marker>\tag important\ gdelta :: "'a::topological_space set \ bool" where "(\n::nat. open (F n)) \ gdelta (\(F ` UNIV))" lemma fsigma_Union_compact: @@ -2100,7 +2100,7 @@ assumes S: "S \ sets lebesgue" and f: "\x. x \ S \ (f has_derivative f' x) (at x within S)" shows "(\x. det(matrix(f' x))) \ borel_measurable (lebesgue_on S)" unfolding det_def - by%unimportant (intro measurable) (auto intro: f borel_measurable_partial_derivatives [OF S]) + by (intro measurable) (auto intro: f borel_measurable_partial_derivatives [OF S]) text\The localisation wrt S uses the same argument for many similar results.\ (*See HOL Light's MEASURABLE_ON_LEBESGUE_MEASURABLE_PREIMAGE_BOREL, etc.*) @@ -2949,7 +2949,7 @@ and intS: "(\x. \det (matrix (g' x))\ *\<^sub>R f(g x)) absolutely_integrable_on S" shows "f absolutely_integrable_on (g ` S)" apply (rule absolutely_integrable_componentwise [OF absolutely_integrable_on_image_real [OF der_g]]) - using%unimportant absolutely_integrable_component [OF intS] by%unimportant auto + using absolutely_integrable_component [OF intS] by auto proposition integral_on_image_ubound: fixes f :: "real^'n::{finite,wellorder} \ real" and g :: "real^'n::_ \ real^'n::_" @@ -2957,7 +2957,7 @@ and "\x. x \ S \ (g has_derivative g' x) (at x within S)" and "(\x. \det (matrix (g' x))\ * f(g x)) integrable_on S" shows "integral (g ` S) f \ integral S (\x. \det (matrix (g' x))\ * f(g x))" - using%unimportant integral_on_image_ubound_nonneg [OF assms] by%unimportant simp + using integral_on_image_ubound_nonneg [OF assms] by simp subsection\Change-of-variables theorem\ @@ -3576,7 +3576,7 @@ and "inj_on g S" shows "f absolutely_integrable_on (g ` S) \ (\x. \det (matrix (g' x))\ *\<^sub>R f(g x)) absolutely_integrable_on S" - using%unimportant assms has_absolute_integral_change_of_variables by%unimportant blast + using assms has_absolute_integral_change_of_variables by blast corollary integral_change_of_variables: fixes f :: "real^'m::{finite,wellorder} \ real^'n" and g :: "real^'m::_ \ real^'m::_" @@ -3586,8 +3586,8 @@ and disj: "(f absolutely_integrable_on (g ` S) \ (\x. \det (matrix (g' x))\ *\<^sub>R f(g x)) absolutely_integrable_on S)" shows "integral (g ` S) f = integral S (\x. \det (matrix (g' x))\ *\<^sub>R f(g x))" - using%unimportant has_absolute_integral_change_of_variables [OF S der_g inj] disj - by%unimportant blast + using has_absolute_integral_change_of_variables [OF S der_g inj] disj + by blast lemma has_absolute_integral_change_of_variables_1: fixes f :: "real \ real^'n::{finite,wellorder}" and g :: "real \ real" @@ -3635,7 +3635,7 @@ and inj: "inj_on g S" shows "(f absolutely_integrable_on g ` S \ (\x. \g' x\ *\<^sub>R f(g x)) absolutely_integrable_on S)" - using%unimportant has_absolute_integral_change_of_variables_1 [OF assms] by%unimportant auto + using has_absolute_integral_change_of_variables_1 [OF assms] by auto subsection\Change of variables for integrals: special case of linear function\