src/HOL/ex/Classical.thy
changeset 15384 b13eb8a8897d
parent 15151 429666b09783
child 16011 237aafbdb1f4
--- a/src/HOL/ex/Classical.thy	Tue Dec 07 16:16:23 2004 +0100
+++ b/src/HOL/ex/Classical.thy	Tue Dec 07 18:10:13 2004 +0100
@@ -720,8 +720,8 @@
        (\<forall>x. (P4 x|P5 x) --> (\<exists>y. Q0 y & R x y))
        --> (\<exists>x y. P0 x & P0 y & (\<exists>z. Q1 z & R y z & R x y))"
 by (tactic{*safe_best_meson_tac 1*})
-    --{*Considerably faster than @{text meson},
-        which does iterative deepening rather than best-first search*}
+    --{*Nearly twice as fast as @{text meson},
+        which performs iterative deepening rather than best-first search*}
 
 text{*The Los problem. Circulated by John Harrison*}
 lemma "(\<forall>x y z. P x y & P y z --> P x z) &
@@ -794,9 +794,9 @@
      and Q: "\<And>U. Q U \<Longrightarrow> False"
      and PQ: "\<And>U.  \<lbrakk>P (f U); \<not> Q (g U)\<rbrakk> \<Longrightarrow> False"
   have cl4: "\<And>U. \<not> Q (g U) \<Longrightarrow> False"
-    by (rule P [BINARY 0 PQ 0])
+    by (rule P [binary 0 PQ 0])
   show "False"
-    by (rule Q [BINARY 0 cl4 0])
+    by (rule Q [binary 0 cl4 0])
 qed
 
 end