diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/ex/Classical.thy --- a/src/HOL/ex/Classical.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/ex/Classical.thy Sat Jan 05 17:24:33 2019 +0100 @@ -428,7 +428,7 @@ lemma "(\x y z. R(x,y) \ R(y,z) \ R(x,z)) \ (\x. \y. R(x,y)) \ \ (\x. P x = (\y. R(x,y) \ \ P y))" -by (tactic\Meson.safe_best_meson_tac @{context} 1\) +by (tactic\Meson.safe_best_meson_tac \<^context> 1\) \ \In contrast, \meson\ is SLOW: 7.6s on griffon\ @@ -722,7 +722,7 @@ (\x y. bird x \ snail y \ \eats x y) \ (\x. (caterpillar x \ snail x) \ (\y. plant y \ eats x y)) \ (\x y. animal x \ animal y \ (\z. grain z \ eats y z \ eats x y))" -by (tactic\Meson.safe_best_meson_tac @{context} 1\) +by (tactic\Meson.safe_best_meson_tac \<^context> 1\) \ \Nearly twice as fast as \meson\, which performs iterative deepening rather than best-first search\