# HG changeset patch # User nipkow # Date 1548424780 -3600 # Node ID 8b47c021666e09cd9c3350939c72fd925597fac6 # Parent c558fef629157c2de8f3b47e3367f4a59988b46a tuned diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Binary_Product_Measure.thy --- a/src/HOL/Analysis/Binary_Product_Measure.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Binary_Product_Measure.thy Fri Jan 25 14:59:40 2019 +0100 @@ -104,13 +104,13 @@ shows "f \ measurable M (M1 \\<^sub>M M2)" using measurable_Pair[OF assms] by simp -lemma (*FIX ME needs a name *) +lemma assumes f[measurable]: "f \ measurable M (N \\<^sub>M P)" shows measurable_fst': "(\x. fst (f x)) \ measurable M N" and measurable_snd': "(\x. snd (f x)) \ measurable M P" by simp_all -lemma (*FIX ME needs a name *) +lemma assumes f[measurable]: "f \ measurable M N" shows measurable_fst'': "(\x. f (fst x)) \ measurable (M \\<^sub>M P) N" and measurable_snd'': "(\x. f (snd x)) \ measurable (P \\<^sub>M M) N" diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Bochner_Integration.thy --- a/src/HOL/Analysis/Bochner_Integration.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Bochner_Integration.thy Fri Jan 25 14:59:40 2019 +0100 @@ -1464,7 +1464,7 @@ using integral_discrete_difference[of X M f g, OF assms] by (metis has_bochner_integral_iff) -lemma (*FIX ME needs name *) +lemma fixes f :: "'a \ 'b::{banach, second_countable_topology}" and w :: "'a \ real" assumes "f \ borel_measurable M" "\i. s i \ borel_measurable M" "integrable M w" assumes lim: "AE x in M. (\i. s i x) \ f x" @@ -1697,7 +1697,7 @@ by (simp_all add: * assms integral_nonneg_AE) qed -lemma (* FIX ME needs name*) +lemma fixes f :: "_ \ _ \ 'a :: {banach, second_countable_topology}" assumes integrable[measurable]: "\i. integrable M (f i)" and summable: "AE x in M. summable (\i. norm (f i x))" @@ -2327,7 +2327,7 @@ qed qed (simp add: f g integrable_density) -lemma (*FIX ME needs name *) +lemma fixes g :: "'a \ real" assumes "f \ borel_measurable M" "AE x in M. 0 \ f x" "g \ borel_measurable M" shows integral_real_density: "integral\<^sup>L (density M f) g = (\ x. f x * g x \M)" @@ -2630,7 +2630,7 @@ by (auto simp: real_integrable_def real_lebesgue_integral_def u) qed -lemma (*FIX ME needs name *) +lemma fixes f :: "nat \ 'a \ real" assumes f: "\i. integrable M (f i)" and mono: "AE x in M. mono (\n. f n x)" and lim: "AE x in M. (\i. f i x) \ u x" @@ -2810,7 +2810,7 @@ qed auto qed -lemma (*FIX ME needs name *) +lemma fixes f :: "real \ real" assumes M: "sets M = sets borel" assumes nonneg: "AE x in M. 0 \ f x" @@ -3154,7 +3154,7 @@ qed qed -lemma (in pair_sigma_finite) (* FIX ME needs name *) +lemma (in pair_sigma_finite) fixes f :: "_ \ _ \ _::{banach, second_countable_topology}" assumes f: "integrable (M1 \\<^sub>M M2) (case_prod f)" shows AE_integrable_fst: "AE x in M1. integrable M2 (\y. f x y)" (is "?AE") @@ -3162,7 +3162,7 @@ and integral_fst: "(\x. (\y. f x y \M2) \M1) = integral\<^sup>L (M1 \\<^sub>M M2) (\(x, y). f x y)" (is "?EQ") using AE_integrable_fst'[OF f] integrable_fst'[OF f] integral_fst'[OF f] by auto -lemma (in pair_sigma_finite) (* FIX ME needs name *) +lemma (in pair_sigma_finite) fixes f :: "_ \ _ \ _::{banach, second_countable_topology}" assumes f[measurable]: "integrable (M1 \\<^sub>M M2) (case_prod f)" shows AE_integrable_snd: "AE y in M2. integrable M1 (\x. f x y)" (is "?AE") diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Borel_Space.thy --- a/src/HOL/Analysis/Borel_Space.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Borel_Space.thy Fri Jan 25 14:59:40 2019 +0100 @@ -797,7 +797,7 @@ finally show ?thesis . qed -lemma (* FIX ME needs name *) +lemma fixes f :: "'a \ 'b::{second_countable_topology, linorder_topology}" assumes f[measurable]: "f \ borel_measurable M" assumes g[measurable]: "g \ borel_measurable M" @@ -929,7 +929,7 @@ "f \ borel_measurable M \ g \ borel_measurable M \ (\x. inf (g x) (f x) :: 'b::{lattice, second_countable_topology, linorder_topology}) \ borel_measurable M" unfolding inf_min by measurable -lemma [measurable (raw)]: (*FIXME needs name *) +lemma [measurable (raw)]: fixes f :: "nat \ 'a \ 'b::{complete_linorder, second_countable_topology, linorder_topology}" assumes "\i. f i \ borel_measurable M" shows borel_measurable_liminf: "(\x. liminf (\i. f i x)) \ borel_measurable M" @@ -1023,7 +1023,7 @@ unfolding box_oc box_co by (auto intro: borel_open borel_closed) -lemma (*FIX ME this has no name *) +lemma fixes i :: "'a::{second_countable_topology, real_inner}" shows hafspace_less_borel: "{x. a < x \ i} \ sets borel" and hafspace_greater_borel: "{x. x \ i < a} \ sets borel" @@ -1551,7 +1551,7 @@ with f H show ?thesis by simp qed -lemma (*FIX ME needs a name *) +lemma fixes f :: "'a \ ereal" assumes f[measurable]: "f \ borel_measurable M" shows borel_measurable_ereal_abs[measurable(raw)]: "(\x. \f x\) \ borel_measurable M" and borel_measurable_ereal_inverse[measurable(raw)]: "(\x. inverse (f x) :: ereal) \ borel_measurable M" diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Change_Of_Vars.thy --- a/src/HOL/Analysis/Change_Of_Vars.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Change_Of_Vars.thy Fri Jan 25 14:59:40 2019 +0100 @@ -963,12 +963,12 @@ then show "f ` S \ lmeasurable" ?M by blast+ qed -lemma (*FIXME needs name? *) +lemma m_diff_image_weak: fixes f :: "real^'n::{finite,wellorder} \ real^'n::_" assumes S: "S \ lmeasurable" and deriv: "\x. x \ S \ (f has_derivative f' x) (at x within S)" and int: "(\x. \det (matrix (f' x))\) integrable_on S" - shows m_diff_image_weak: "f ` S \ lmeasurable \ measure lebesgue (f ` S) \ integral S (\x. \det (matrix (f' x))\)" + shows "f ` S \ lmeasurable \ measure lebesgue (f ` S) \ integral S (\x. \det (matrix (f' x))\)" proof - let ?\ = "measure lebesgue" have aint_S: "(\x. \det (matrix (f' x))\) absolutely_integrable_on S" @@ -1161,7 +1161,7 @@ qed -theorem(* FIXME needs name? *) +theorem fixes f :: "real^'n::{finite,wellorder} \ real^'n::_" assumes S: "S \ sets lebesgue" and deriv: "\x. x \ S \ (f has_derivative f' x) (at x within S)" diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Finite_Product_Measure.thy --- a/src/HOL/Analysis/Finite_Product_Measure.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Finite_Product_Measure.thy Fri Jan 25 14:59:40 2019 +0100 @@ -397,7 +397,7 @@ apply (auto intro!: arg_cong2[where f=sigma_sets]) done -lemma (*FIX ME needs name *) +lemma shows space_PiM_empty: "space (Pi\<^sub>M {} M) = {\k. undefined}" and sets_PiM_empty: "sets (Pi\<^sub>M {} M) = { {}, {\k. undefined} }" by (simp_all add: space_PiM sets_PiM_single image_constant sigma_sets_empty_eq) diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Homeomorphism.thy --- a/src/HOL/Analysis/Homeomorphism.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Homeomorphism.thy Fri Jan 25 14:59:40 2019 +0100 @@ -278,7 +278,7 @@ qed qed -proposition (*FIXME needs name *) +proposition fixes S :: "'a::euclidean_space set" assumes "compact S" and 0: "0 \ rel_interior S" and star: "\x. x \ S \ open_segment 0 x \ rel_interior S" @@ -540,7 +540,7 @@ done qed -corollary (* FIXME needs name *) +corollary fixes S :: "'a::euclidean_space set" assumes "compact S" and a: "a \ rel_interior S" and star: "\x. x \ S \ open_segment a x \ rel_interior S" diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Poly_Roots.thy --- a/src/HOL/Analysis/Poly_Roots.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Poly_Roots.thy Fri Jan 25 14:59:40 2019 +0100 @@ -182,7 +182,7 @@ qed simp qed simp -corollary (*FIX ME needs name *) +corollary fixes c :: "nat \ 'a::{comm_ring,real_normed_div_algebra}" assumes "\k. k \ n \ c k \ 0" shows polyfun_rootbound_finite: "finite {z. (\i\n. c i * z^i) = 0}" diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Radon_Nikodym.thy --- a/src/HOL/Analysis/Radon_Nikodym.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Radon_Nikodym.thy Fri Jan 25 14:59:40 2019 +0100 @@ -1022,7 +1022,7 @@ by simp qed -lemma (in sigma_finite_measure) (* FIXME needs name*) +lemma (in sigma_finite_measure) assumes N: "sigma_finite_measure N" and ac: "absolutely_continuous M N" "sets N = sets M" and f: "f \ borel_measurable M" shows RN_deriv_integrable: "integrable N f \ diff -r c558fef62915 -r 8b47c021666e src/HOL/Analysis/Regularity.thy --- a/src/HOL/Analysis/Regularity.thy Fri Jan 25 13:19:16 2019 +0100 +++ b/src/HOL/Analysis/Regularity.thy Fri Jan 25 14:59:40 2019 +0100 @@ -9,7 +9,7 @@ imports Measure_Space Borel_Space begin -theorem (*FIX needs name *) +theorem fixes M::"'a::{second_countable_topology, complete_space} measure" assumes sb: "sets M = sets borel" assumes "emeasure M (space M) \ \"