# HG changeset patch # User wenzelm # Date 1452027441 -3600 # Node ID bf3d9f1134748f22ee01ad17cb6d153759f883b8 # Parent 4e6e850e97c252f97798a16c1bae1fbc4ef1c128 isabelle update_cartouches -c -t; diff -r 4e6e850e97c2 -r bf3d9f113474 src/HOL/Library/Nonpos_Ints.thy --- a/src/HOL/Library/Nonpos_Ints.thy Tue Jan 05 21:55:40 2016 +0100 +++ b/src/HOL/Library/Nonpos_Ints.thy Tue Jan 05 21:57:21 2016 +0100 @@ -46,7 +46,7 @@ hence "(of_int m :: 'a) = of_nat n" by simp also have "... = of_int (int n)" by simp finally have "m = int n" by (subst (asm) of_int_eq_iff) - with `m \ 0` show "n = 0" by auto + with \m \ 0\ show "n = 0" by auto qed simp lemma nonpos_Ints_of_int: "n \ 0 \ of_int n \ \\<^sub>\\<^sub>0" @@ -84,10 +84,10 @@ proof assume "of_real x \ (\\<^sub>\\<^sub>0 :: 'a set)" then obtain n where "(of_real x :: 'a) = of_int n" "n \ 0" by (erule nonpos_Ints_cases) - note `of_real x = of_int n` + note \of_real x = of_int n\ also have "of_int n = of_real (of_int n)" by (rule of_real_of_int_eq [symmetric]) finally have "x = of_int n" by (subst (asm) of_real_eq_iff) - with `n \ 0` show "x \ \\<^sub>\\<^sub>0" by (simp add: nonpos_Ints_of_int) + with \n \ 0\ show "x \ \\<^sub>\\<^sub>0" by (simp add: nonpos_Ints_of_int) qed (auto elim!: nonpos_Ints_cases intro!: nonpos_Ints_of_int) lemma nonpos_Ints_altdef: "\\<^sub>\\<^sub>0 = {n \ \. (n :: 'a :: linordered_idom) \ 0}" diff -r 4e6e850e97c2 -r bf3d9f113474 src/HOL/Library/Poly_Deriv.thy --- a/src/HOL/Library/Poly_Deriv.thy Tue Jan 05 21:55:40 2016 +0100 +++ b/src/HOL/Library/Poly_Deriv.thy Tue Jan 05 21:57:21 2016 +0100 @@ -167,7 +167,7 @@ proof - assume "p\0" then obtain n1 where gte_lcoeff:"\x\n1. lead_coeff p \ poly p x" using that pCons by auto - have gt_0:"lead_coeff p >0" using pCons(3) `p\0` by auto + have gt_0:"lead_coeff p >0" using pCons(3) \p\0\ by auto def n\"max n1 (1+ \a\/(lead_coeff p))" show ?thesis proof (rule_tac x=n in exI,rule,rule) @@ -176,9 +176,9 @@ using gte_lcoeff unfolding n_def by auto hence " \a\/(lead_coeff p) \ \a\/(poly p x)" and "poly p x>0" using gt_0 by (intro frac_le,auto) - hence "x\1+ \a\/(poly p x)" using `n\x`[unfolded n_def] by auto + hence "x\1+ \a\/(poly p x)" using \n\x\[unfolded n_def] by auto thus "lead_coeff (pCons a p) \ poly (pCons a p) x" - using `lead_coeff p \ poly p x` `poly p x>0` `p\0` + using \lead_coeff p \ poly p x\ \poly p x>0\ \p\0\ by (auto simp add:field_simps) qed qed diff -r 4e6e850e97c2 -r bf3d9f113474 src/HOL/Library/Polynomial.thy --- a/src/HOL/Library/Polynomial.thy Tue Jan 05 21:55:40 2016 +0100 +++ b/src/HOL/Library/Polynomial.thy Tue Jan 05 21:57:21 2016 +0100 @@ -475,7 +475,7 @@ coeff ?p' 0 * x^0 + (\i\degree p. coeff ?p' (Suc i) * x^Suc i)" by (simp add: field_simps setsum_right_distrib coeff_pCons) also note setsum_atMost_Suc_shift[symmetric] - also note degree_pCons_eq[OF `p \ 0`, of a, symmetric] + also note degree_pCons_eq[OF \p \ 0\, of a, symmetric] finally show ?thesis . qed simp qed simp @@ -2145,19 +2145,19 @@ next case False assume "degree (q * pcompose p q) = 0" hence "degree q=0 \ pcompose p q=0" by (auto simp add:degree_mult_eq_0) - moreover have "\pcompose p q=0;degree q\0\ \ False" using pCons.hyps(2) `p\0` + moreover have "\pcompose p q=0;degree q\0\ \ False" using pCons.hyps(2) \p\0\ proof - assume "pcompose p q=0" "degree q\0" hence "degree p=0" using pCons.hyps(2) by auto then obtain a1 where "p=[:a1:]" by (metis degree_pCons_eq_if old.nat.distinct(2) pCons_cases) - thus False using `pcompose p q=0` `p\0` by auto + thus False using \pcompose p q=0\ \p\0\ by auto qed ultimately have "degree (pCons a p) * degree q=0" by auto moreover have "degree (pcompose (pCons a p) q) = 0" proof - have" 0 = max (degree [:a:]) (degree (q*pcompose p q))" - using `degree (q * pcompose p q) = 0` by simp + using \degree (q * pcompose p q) = 0\ by simp also have "... \ degree ([:a:] + q * pcompose p q)" by (rule degree_add_le_max) finally show ?thesis by (auto simp add:pcompose_pCons) @@ -2172,7 +2172,7 @@ unfolding pcompose_pCons using degree_add_eq_right[of "[:a:]" ] asm by auto thus ?thesis - using pCons.hyps(2) degree_mult_eq[OF `q\0` `pcompose p q\0`] by auto + using pCons.hyps(2) degree_mult_eq[OF \q\0\ \pcompose p q\0\] by auto qed ultimately show ?case by blast qed @@ -2186,11 +2186,11 @@ then obtain a where "p=[:a:]" by (metis degree_pCons_eq_if gr0_conv_Suc neq0_conv pCons_cases) hence "a=0" using assms(1) by auto - thus ?thesis using `p=[:a:]` by simp + thus ?thesis using \p=[:a:]\ by simp qed -subsection {* Leading coefficient *} +subsection \Leading coefficient\ definition lead_coeff:: "'a::zero poly \ 'a" where "lead_coeff p= coeff p (degree p)" @@ -2232,7 +2232,7 @@ proof - assume "degree ( q * pcompose p q) = 0" hence "pcompose p q = 0" by (metis assms degree_0 degree_mult_eq_0 neq0_conv) - hence "p=0" using pcompose_eq_0[OF _ `degree q > 0`] by simp + hence "p=0" using pcompose_eq_0[OF _ \degree q > 0\] by simp thus ?thesis by auto qed moreover have "degree ( q * pcompose p q) > 0 \ ?case" diff -r 4e6e850e97c2 -r bf3d9f113474 src/HOL/Multivariate_Analysis/Gamma.thy --- a/src/HOL/Multivariate_Analysis/Gamma.thy Tue Jan 05 21:55:40 2016 +0100 +++ b/src/HOL/Multivariate_Analysis/Gamma.thy Tue Jan 05 21:57:21 2016 +0100 @@ -169,7 +169,7 @@ also have "\ \ dist z (of_int n)" using round_Re_minimises_norm[of z] by (simp add: dist_complex_def) finally have "dist t (of_int n) > 0" by simp - with `t = of_int n` show False by simp + with \t = of_int n\ show False by simp qed lemma no_nonpos_Int_in_ball': @@ -377,7 +377,7 @@ finally have "of_nat N \ 2 * (norm z + d)" . moreover have "N \ 2" "N \ M" unfolding N_def by simp_all moreover have "(\k=m..n. 1/(of_nat k)\<^sup>2) < e'" if "m \ N" for m n - using M[OF order.trans[OF `N \ M` that]] unfolding real_norm_def + using M[OF order.trans[OF \N \ M\ that]] unfolding real_norm_def by (subst (asm) abs_of_nonneg) (auto intro: setsum_nonneg simp: divide_simps) moreover note calculation } note N = this @@ -1959,7 +1959,7 @@ let ?h = "\z::complex. (of_real pi * cot (of_real pi*z) + Digamma z - Digamma (1 - z))" def h \ "\z::complex. if z \ \ then 0 else ?h z" - -- \@{term g} is periodic with period 1.\ + \ \@{term g} is periodic with period 1.\ interpret g: periodic_fun_simple' g proof fix z :: complex @@ -1979,7 +1979,7 @@ qed (simp add: g_def) qed - -- \@{term g} is entire.\ + \ \@{term g} is entire.\ have g_g': "(g has_field_derivative (h z * g z)) (at z)" for z :: complex proof (cases "z \ \") let ?h' = "\z. Beta z (1 - z) * ((Digamma z - Digamma (1 - z)) * sin (z * of_real pi) + @@ -2204,7 +2204,7 @@ show ?thesis proof (cases "z \ \") case False - with `g z = pi` show ?thesis by (auto simp: g_def divide_simps) + with \g z = pi\ show ?thesis by (auto simp: g_def divide_simps) next case True then obtain n where n: "z = of_int n" by (elim Ints_cases) diff -r 4e6e850e97c2 -r bf3d9f113474 src/HOL/Multivariate_Analysis/Summation.thy --- a/src/HOL/Multivariate_Analysis/Summation.thy Tue Jan 05 21:55:40 2016 +0100 +++ b/src/HOL/Multivariate_Analysis/Summation.thy Tue Jan 05 21:57:21 2016 +0100 @@ -141,7 +141,7 @@ with l obtain l' where l': "l = ereal l'" by (cases l) simp_all def c \ "(1 - l') / 2" - from l and `l \ 0` have c: "l + c > l" "l' + c \ 0" "l' + c < 1" unfolding c_def + from l and \l \ 0\ have c: "l + c > l" "l' + c \ 0" "l' + c < 1" unfolding c_def by (simp_all add: field_simps l') have "\C>l. eventually (\n. ereal (root n (norm (f n))) < C) sequentially" by (subst Limsup_le_iff[symmetric]) (simp add: l_def)