diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/Bali/Example.thy --- a/src/HOL/Bali/Example.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/Bali/Example.thy Sat Jan 05 17:24:33 2019 +0100 @@ -898,7 +898,7 @@ declare member_is_static_simp [simp] declare wt.Skip [rule del] wt.Init [rule del] -ML \ML_Thms.bind_thms ("wt_intros", map (rewrite_rule @{context} @{thms id_def}) @{thms wt.intros})\ +ML \ML_Thms.bind_thms ("wt_intros", map (rewrite_rule \<^context> @{thms id_def}) @{thms wt.intros})\ lemmas wtIs = wt_Call wt_Super wt_FVar wt_StatRef wt_intros lemmas daIs = assigned.select_convs da_Skip da_NewC da_Lit da_Super da.intros @@ -1192,8 +1192,8 @@ Base_foo_defs [simp] ML \ML_Thms.bind_thms ("eval_intros", map - (simplify (@{context} delsimps @{thms Skip_eq} addsimps @{thms lvar_def}) o - rewrite_rule @{context} [@{thm assign_def}, @{thm Let_def}]) @{thms eval.intros})\ + (simplify (\<^context> delsimps @{thms Skip_eq} addsimps @{thms lvar_def}) o + rewrite_rule \<^context> [@{thm assign_def}, @{thm Let_def}]) @{thms eval.intros})\ lemmas eval_Is = eval_Init eval_StatRef AbruptIs eval_intros axiomatization