src/HOL/Tools/Meson/meson_clausify.ML
changeset 67091 1393c2340eec
parent 61268 abe08fb15a12
child 67149 e61557884799
--- a/src/HOL/Tools/Meson/meson_clausify.ML	Sun Nov 26 13:19:52 2017 +0100
+++ b/src/HOL/Tools/Meson/meson_clausify.ML	Sun Nov 26 21:08:32 2017 +0100
@@ -292,7 +292,7 @@
 fun ss_only ths ctxt = clear_simpset (put_simpset HOL_basic_ss ctxt) addsimps ths
 
 val cheat_choice =
-  @{prop "ALL x. EX y. Q x y ==> EX f. ALL x. Q x (f x)"}
+  @{prop "\<forall>x. \<exists>y. Q x y \<Longrightarrow> \<exists>f. \<forall>x. Q x (f x)"}
   |> Logic.varify_global
   |> Skip_Proof.make_thm @{theory}