# HG changeset patch # User wenzelm # Date 1519161923 -3600 # Node ID 00c43648839802ef0899ecd019427a0e6d7ac719 # Parent b5058ba95e32133e449fcb86b2bfdf86d5e5fc09 tuned proofs -- prefer explicit names for facts from 'interpret'; diff -r b5058ba95e32 -r 00c436488398 src/HOL/Analysis/Brouwer_Fixpoint.thy --- a/src/HOL/Analysis/Brouwer_Fixpoint.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/Analysis/Brouwer_Fixpoint.thy Tue Feb 20 22:25:23 2018 +0100 @@ -941,8 +941,8 @@ for i j interpret b: kuhn_simplex p n base ?upd "f' ` {.. n}" proof - show "base \ {.. {.. i" then show "base i = p" by fact } + show "base \ {.. {.. i" then show "base i = p" by (rule base_out) } show "bij_betw ?upd {.. I" then show "\' (G i) = \ i" using \' by (auto intro!: inj sel) } show "G ` I \ Pow \" - by fact + by (rule space_closed) then show "positive (sets M) \'" "countably_additive (sets M) \'" using \' by (simp_all add: M sets_extend_measure measure_space_def) qed fact diff -r b5058ba95e32 -r 00c436488398 src/HOL/Analysis/Derivative.thy --- a/src/HOL/Analysis/Derivative.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/Analysis/Derivative.thy Tue Feb 20 22:25:23 2018 +0100 @@ -1088,7 +1088,7 @@ interpret bounded_linear "(f' ?u)" using u by (auto intro!: has_derivative_bounded_linear assms(2)[rule_format] *) have "norm (f' ?u (y - x)) \ onorm (f' ?u) * norm (y - x)" - by (rule onorm) fact + by (rule onorm) (rule bounded_linear) also have "onorm (f' ?u) \ B" using u by (auto intro!: assms(3)[rule_format] *) finally have "norm ((f' ?u) (y - x)) \ B * norm (x - y)" diff -r b5058ba95e32 -r 00c436488398 src/HOL/HOLCF/ConvexPD.thy --- a/src/HOL/HOLCF/ConvexPD.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/HOLCF/ConvexPD.thy Tue Feb 20 22:25:23 2018 +0100 @@ -430,8 +430,8 @@ assumes "finite_deflation d" shows "finite_deflation (convex_map\d)" proof (rule finite_deflation_intro) interpret d: finite_deflation d by fact - have "deflation d" by fact - thus "deflation (convex_map\d)" by (rule deflation_convex_map) + from d.deflation_axioms show "deflation (convex_map\d)" + by (rule deflation_convex_map) have "finite (range (\x. d\x))" by (rule d.finite_range) hence "finite (Rep_compact_basis -` range (\x. d\x))" by (rule finite_vimageI, simp add: inj_on_def Rep_compact_basis_inject) diff -r b5058ba95e32 -r 00c436488398 src/HOL/HOLCF/LowerPD.thy --- a/src/HOL/HOLCF/LowerPD.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/HOLCF/LowerPD.thy Tue Feb 20 22:25:23 2018 +0100 @@ -423,8 +423,8 @@ assumes "finite_deflation d" shows "finite_deflation (lower_map\d)" proof (rule finite_deflation_intro) interpret d: finite_deflation d by fact - have "deflation d" by fact - thus "deflation (lower_map\d)" by (rule deflation_lower_map) + from d.deflation_axioms show "deflation (lower_map\d)" + by (rule deflation_lower_map) have "finite (range (\x. d\x))" by (rule d.finite_range) hence "finite (Rep_compact_basis -` range (\x. d\x))" by (rule finite_vimageI, simp add: inj_on_def Rep_compact_basis_inject) diff -r b5058ba95e32 -r 00c436488398 src/HOL/HOLCF/Map_Functions.thy --- a/src/HOL/HOLCF/Map_Functions.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/HOLCF/Map_Functions.thy Tue Feb 20 22:25:23 2018 +0100 @@ -92,8 +92,7 @@ proof (rule finite_deflation_intro) interpret d1: finite_deflation d1 by fact interpret d2: finite_deflation d2 by fact - have "deflation d1" and "deflation d2" by fact+ - then show "deflation (cfun_map\d1\d2)" + from d1.deflation_axioms d2.deflation_axioms show "deflation (cfun_map\d1\d2)" by (rule deflation_cfun_map) have "finite (range (\f. cfun_map\d1\d2\f))" using d1.finite_range d2.finite_range @@ -158,8 +157,8 @@ proof (rule finite_deflation_intro) interpret d1: finite_deflation d1 by fact interpret d2: finite_deflation d2 by fact - have "deflation d1" and "deflation d2" by fact+ - then show "deflation (prod_map\d1\d2)" by (rule deflation_prod_map) + from d1.deflation_axioms d2.deflation_axioms show "deflation (prod_map\d1\d2)" + by (rule deflation_prod_map) have "{p. prod_map\d1\d2\p = p} \ {x. d1\x = x} \ {y. d2\y = y}" by auto then show "finite {p. prod_map\d1\d2\p = p}" @@ -204,8 +203,7 @@ shows "finite_deflation (u_map\d)" proof (rule finite_deflation_intro) interpret d: finite_deflation d by fact - have "deflation d" by fact - then show "deflation (u_map\d)" + from d.deflation_axioms show "deflation (u_map\d)" by (rule deflation_u_map) have "{x. u_map\d\x = x} \ insert \ ((\x. up\x) ` {x. d\x = x})" by (rule subsetI, case_tac x, simp_all) @@ -284,8 +282,7 @@ proof (rule finite_deflation_intro) interpret d1: finite_deflation d1 by fact interpret d2: finite_deflation d2 by fact - have "deflation d1" and "deflation d2" by fact+ - then show "deflation (sprod_map\d1\d2)" + from d1.deflation_axioms d2.deflation_axioms show "deflation (sprod_map\d1\d2)" by (rule deflation_sprod_map) have "{x. sprod_map\d1\d2\x = x} \ insert \ ((\(x, y). (:x, y:)) ` ({x. d1\x = x} \ {y. d2\y = y}))" @@ -369,8 +366,7 @@ proof (rule finite_deflation_intro) interpret d1: finite_deflation d1 by fact interpret d2: finite_deflation d2 by fact - have "deflation d1" and "deflation d2" by fact+ - then show "deflation (ssum_map\d1\d2)" + from d1.deflation_axioms d2.deflation_axioms show "deflation (ssum_map\d1\d2)" by (rule deflation_ssum_map) have "{x. ssum_map\d1\d2\x = x} \ (\x. sinl\x) ` {x. d1\x = x} \ @@ -442,8 +438,7 @@ proof (intro finite_deflation_intro) interpret d1: finite_deflation d1 by fact interpret d2: finite_deflation d2 by fact - have "deflation d1" and "deflation d2" by fact+ - then show "deflation (sfun_map\d1\d2)" + from d1.deflation_axioms d2.deflation_axioms show "deflation (sfun_map\d1\d2)" by (rule deflation_sfun_map) from assms have "finite_deflation (cfun_map\d1\d2)" by (rule finite_deflation_cfun_map) diff -r b5058ba95e32 -r 00c436488398 src/HOL/HOLCF/UpperPD.thy --- a/src/HOL/HOLCF/UpperPD.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/HOLCF/UpperPD.thy Tue Feb 20 22:25:23 2018 +0100 @@ -416,8 +416,8 @@ assumes "finite_deflation d" shows "finite_deflation (upper_map\d)" proof (rule finite_deflation_intro) interpret d: finite_deflation d by fact - have "deflation d" by fact - thus "deflation (upper_map\d)" by (rule deflation_upper_map) + from d.deflation_axioms show "deflation (upper_map\d)" + by (rule deflation_upper_map) have "finite (range (\x. d\x))" by (rule d.finite_range) hence "finite (Rep_compact_basis -` range (\x. d\x))" by (rule finite_vimageI, simp add: inj_on_def Rep_compact_basis_inject) diff -r b5058ba95e32 -r 00c436488398 src/HOL/Library/RBT_Set.thy --- a/src/HOL/Library/RBT_Set.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/Library/RBT_Set.thy Tue Feb 20 22:25:23 2018 +0100 @@ -474,7 +474,7 @@ proof - interpret comp_fun_idem Set.insert by (fact comp_fun_idem_insert) - from finite_fold_fold_keys[OF \comp_fun_commute Set.insert\] + from finite_fold_fold_keys[OF comp_fun_commute_axioms] show ?thesis by (auto simp add: union_fold_insert) qed @@ -487,7 +487,7 @@ proof - interpret comp_fun_idem Set.remove by (fact comp_fun_idem_remove) - from finite_fold_fold_keys[OF \comp_fun_commute Set.remove\] + from finite_fold_fold_keys[OF comp_fun_commute_axioms] show ?thesis by (auto simp add: minus_fold_remove) qed diff -r b5058ba95e32 -r 00c436488398 src/HOL/Probability/Levy.thy --- a/src/HOL/Probability/Levy.thy Tue Feb 20 22:04:04 2018 +0100 +++ b/src/HOL/Probability/Levy.thy Tue Feb 20 22:25:23 2018 +0100 @@ -219,7 +219,7 @@ { fix \ :: real assume "\ > 0" have "(?D \ 0) at_bot" - using \(cdf M1 \ 0) at_bot\ \(cdf M2 \ 0) at_bot\ by (intro tendsto_eq_intros) auto + using M1.cdf_lim_at_bot M2.cdf_lim_at_bot by (intro tendsto_eq_intros) auto then have "eventually (\y. ?D y < \ / 2 \ y \ x) at_bot" using \\ > 0\ by (simp only: tendsto_iff dist_real_def diff_0_right eventually_conj eventually_le_at_bot abs_idempotent) then obtain M where "\y. y \ M \ ?D y < \ / 2" "M \ x"