# HG changeset patch # User huffman # Date 1522264401 25200 # Node ID 732c0b0594635d62a359de0c6617214c931773bf # Parent 55f00429da84ad92f975ee5b08d999e62c503bf2 tuned proofs and generalized some lemmas about limits diff -r 55f00429da84 -r 732c0b059463 src/HOL/Limits.thy --- a/src/HOL/Limits.thy Wed Mar 28 12:12:19 2018 -0700 +++ b/src/HOL/Limits.thy Wed Mar 28 12:13:21 2018 -0700 @@ -175,16 +175,12 @@ assumes "eventually (\n. norm (f n) \ norm (g n)) sequentially" "Bseq g" shows "Bseq f" proof - - from assms(1) obtain N where N: "\n. n \ N \ norm (f n) \ norm (g n)" - by (auto simp: eventually_at_top_linorder) - moreover from assms(2) obtain K where K: "\n. norm (g n) \ K" - by (blast elim!: BseqE) - ultimately have "norm (f n) \ max K (Max {norm (f n) |n. n < N})" for n - apply (cases "n < N") - subgoal by (rule max.coboundedI2, rule Max.coboundedI) auto - subgoal by (rule max.coboundedI1) (force intro: order.trans[OF N K]) - done - then show ?thesis by (blast intro: BseqI') + from assms(2) obtain K where "0 < K" and "eventually (\n. norm (g n) \ K) sequentially" + unfolding Bfun_def by fast + with assms(1) have "eventually (\n. norm (f n) \ K) sequentially" + by (fast elim: eventually_elim2 order_trans) + with `0 < K` show "Bseq f" + unfolding Bfun_def by fast qed lemma lemma_NBseq_def: "(\K > 0. \n. norm (X n) \ K) \ (\N. \n. norm (X n) \ real(Suc N))" @@ -2264,12 +2260,6 @@ subsection \Power Sequences\ -text \ - The sequence @{term "x^n"} tends to 0 if @{term "0\x"} and @{term - "x<1"}. Proof will use (NS) Cauchy equivalence for convergence and - also fact that bounded and monotonic sequence converges. -\ - lemma Bseq_realpow: "0 \ x \ x \ 1 \ Bseq (\n. x ^ n)" for x :: real apply (simp add: Bseq_def) @@ -2713,14 +2703,14 @@ qed lemma open_Collect_positive: - fixes f :: "'a::t2_space \ real" + fixes f :: "'a::topological_space \ real" assumes f: "continuous_on s f" shows "\A. open A \ A \ s = {x\s. 0 < f x}" using continuous_on_open_invariant[THEN iffD1, OF f, rule_format, of "{0 <..}"] by (auto simp: Int_def field_simps) lemma open_Collect_less_Int: - fixes f g :: "'a::t2_space \ real" + fixes f g :: "'a::topological_space \ real" assumes f: "continuous_on s f" and g: "continuous_on s g" shows "\A. open A \ A \ s = {x\s. f x < g x}"