# HG changeset patch # User wenzelm # Date 1519489295 -3600 # Node ID 5a1b299fe4af77c7ceabf068df0eff2ddcfa94e4 # Parent 3f611f444c2da26486d7e735e185afc93dc312dd more symbols; diff -r 3f611f444c2d -r 5a1b299fe4af src/HOL/Library/While_Combinator.thy --- a/src/HOL/Library/While_Combinator.thy Fri Feb 23 21:46:30 2018 +0100 +++ b/src/HOL/Library/While_Combinator.thy Sat Feb 24 17:21:35 2018 +0100 @@ -68,7 +68,7 @@ define k where "k = (LEAST k. \ b ((c ^^ k) s))" from assms have t: "t = (c ^^ k) s" by (simp add: while_option_def k_def split: if_splits) - have 1: "ALL ii k" then have "P ((c ^^ i) s)" diff -r 3f611f444c2d -r 5a1b299fe4af src/HOL/List.thy --- a/src/HOL/List.thy Fri Feb 23 21:46:30 2018 +0100 +++ b/src/HOL/List.thy Sat Feb 24 17:21:35 2018 +0100 @@ -1716,7 +1716,7 @@ lemma list_eq_iff_nth_eq: - "(xs = ys) = (length xs = length ys \ (ALL i (\i!i < length xs. P(xs!i); x \ set xs\ \ P x" + "\\i < length xs. P(xs!i); x \ set xs\ \ P x" by (auto simp add: set_conv_nth) lemma all_set_conv_all_nth: @@ -3150,7 +3150,7 @@ done lemma nth_equalityI: - "[| length xs = length ys; ALL i < length xs. xs!i = ys!i |] ==> xs = ys" + "[| length xs = length ys; \i < length xs. xs!i = ys!i |] ==> xs = ys" by (frule nth_take_lemma [OF le_refl eq_imp_le]) simp_all lemma map_nth: diff -r 3f611f444c2d -r 5a1b299fe4af src/HOL/MicroJava/DFA/Typing_Framework.thy --- a/src/HOL/MicroJava/DFA/Typing_Framework.thy Fri Feb 23 21:46:30 2018 +0100 +++ b/src/HOL/MicroJava/DFA/Typing_Framework.thy Sat Feb 24 17:21:35 2018 +0100 @@ -18,12 +18,12 @@ "stable r step ss p == \(q,s')\set(step p (ss!p)). s' <=_r ss!q" definition stables :: "'s ord \ 's step_type \ 's list \ bool" where -"stables r step ss == !pp 's \ 's step_type \ 's list \ bool" where "wt_step r T step ts == - !pp 's \ 's step_type \ nat \ 's set \ ('s list \ 's list) \ bool" where diff -r 3f611f444c2d -r 5a1b299fe4af src/HOL/UNITY/Comp/Alloc.thy --- a/src/HOL/UNITY/Comp/Alloc.thy Fri Feb 23 21:46:30 2018 +0100 +++ b/src/HOL/UNITY/Comp/Alloc.thy Sat Feb 24 17:21:35 2018 +0100 @@ -943,7 +943,7 @@ done text\progress (2), step 4\ -lemma System_Bounded_allocAsk: "System \ Always {s. ALL i Always {s. \ielt \ set ((sub i o allocAsk) s). elt \ NbT}" apply (auto simp add: Collect_all_imp_eq) apply (tactic \resolve_tac @{context} [Always_Int_rule [@{thm Always_allocAsk_le_ask},