# HG changeset patch # User wenzelm # Date 1354018949 -3600 # Node ID 8b0fdeeefef7232b8818cca90bf56e08c70344cf # Parent 019d642d422d2bc796bb373d2c72e44235948516 eliminated some improper identifiers; diff -r 019d642d422d -r 8b0fdeeefef7 src/HOL/Decision_Procs/MIR.thy --- a/src/HOL/Decision_Procs/MIR.thy Tue Nov 27 10:56:31 2012 +0100 +++ b/src/HOL/Decision_Procs/MIR.thy Tue Nov 27 13:22:29 2012 +0100 @@ -5010,7 +5010,7 @@ from alluopairs_set1[where xs="?U"] have UpU: "set ?Up \ (set ?U \ set ?U)" by simp from \_l[OF lq] have U_l: "\ (t,n) \ set ?U. numbound0 t \ n > 0" . from U_l UpU - have Up_: "\ ((t,n),(s,m)) \ set ?Up. numbound0 t \ n> 0 \ numbound0 s \ m > 0" by auto + have "\ ((t,n),(s,m)) \ set ?Up. numbound0 t \ n> 0 \ numbound0 s \ m > 0" by auto hence Snb: "\ (t,n) \ set ?S. numbound0 t \ n > 0 " by (auto simp add: mult_pos_pos) have Y_l: "\ (t,n) \ set ?Y. numbound0 t \ n > 0" diff -r 019d642d422d -r 8b0fdeeefef7 src/HOL/Multivariate_Analysis/Integration.thy --- a/src/HOL/Multivariate_Analysis/Integration.thy Tue Nov 27 10:56:31 2012 +0100 +++ b/src/HOL/Multivariate_Analysis/Integration.thy Tue Nov 27 13:22:29 2012 +0100 @@ -996,9 +996,9 @@ thus ?thesis apply- apply(rule that[of q]) unfolding True by auto next case False note p = division_ofD[OF assms(1)] have *:"\k\p. \q. q division_of {a..b} \ k\q" proof case goal1 - guess c using p(4)[OF goal1] .. then guess d .. note cd_ = this - have *:"{c..d} \ {a..b}" "{c..d} \ {}" using p(2,3)[OF goal1, unfolded cd_] using assms(2) by auto - guess q apply(rule partial_division_extend_1[OF *]) . thus ?case unfolding cd_ by auto qed + guess c using p(4)[OF goal1] .. then guess d .. note "cd" = this + have *:"{c..d} \ {a..b}" "{c..d} \ {}" using p(2,3)[OF goal1, unfolded "cd"] using assms(2) by auto + guess q apply(rule partial_division_extend_1[OF *]) . thus ?case unfolding "cd" by auto qed guess q using bchoice[OF *] .. note q = conjunctD2[OF this[rule_format]] have "\x. x\p \ \d. d division_of \(q x - {x})" apply(rule,rule_tac p="q x" in division_of_subset) proof- fix x assume x:"x\p" show "q x division_of \q x" apply-apply(rule division_ofI) diff -r 019d642d422d -r 8b0fdeeefef7 src/HOL/Proofs/Lambda/StrongNorm.thy --- a/src/HOL/Proofs/Lambda/StrongNorm.thy Tue Nov 27 10:56:31 2012 +0100 +++ b/src/HOL/Proofs/Lambda/StrongNorm.thy Tue Nov 27 13:22:29 2012 +0100 @@ -102,7 +102,7 @@ assume uIT: "IT u" assume uT: "e \ u : T" { - case (Var rs n e_ T'_ u_ i_) + case (Var rs n e1 T'1 u1 i1) assume nT: "e\i:T\ \ Var n \\ rs : T'" let ?ty = "\t. \T'. e\i:T\ \ t : T'" let ?R = "\t. \e T' u i. @@ -210,13 +210,13 @@ with False show ?thesis by (auto simp add: subst_Var) qed next - case (Lambda r e_ T'_ u_ i_) + case (Lambda r e1 T'1 u1 i1) assume "e\i:T\ \ Abs r : T'" and "\e T' u i. PROP ?Q r e T' u i T" with uIT uT show "IT (Abs r[u/i])" by fastforce next - case (Beta r a as e_ T'_ u_ i_) + case (Beta r a as e1 T'1 u1 i1) assume T: "e\i:T\ \ Abs r \ a \\ as : T'" assume SI1: "\e T' u i. PROP ?Q (r[a/0] \\ as) e T' u i T" assume SI2: "\e T' u i. PROP ?Q a e T' u i T" diff -r 019d642d422d -r 8b0fdeeefef7 src/HOL/Proofs/Lambda/WeakNorm.thy --- a/src/HOL/Proofs/Lambda/WeakNorm.thy Tue Nov 27 10:56:31 2012 +0100 +++ b/src/HOL/Proofs/Lambda/WeakNorm.thy Tue Nov 27 13:22:29 2012 +0100 @@ -76,7 +76,7 @@ proof induct fix e T' u i assume uNF: "NF u" and uT: "e \ u : T" { - case (App ts x e_ T'_ u_ i_) + case (App ts x e1 T'1 u1 i1) assume "e\i:T\ \ Var x \\ ts : T'" then obtain Us where varT: "e\i:T\ \ Var x : Us \ T'" @@ -187,7 +187,7 @@ qed qed next - case (Abs r e_ T'_ u_ i_) + case (Abs r e1 T'1 u1 i1) assume absT: "e\i:T\ \ Abs r : T'" then obtain R S where "e\0:R\\Suc i:T\ \ r : S" by (rule abs_typeE) simp moreover have "NF (lift u 0)" using `NF u` by (rule lift_NF)