src/HOL/TPTP/TPTP_Parser/tptp_reconstruct_library.ML
changeset 67613 ce654b0e6d69
parent 67399 eab6ce8368fa
child 69597 ff784d5a5bfb
--- a/src/HOL/TPTP/TPTP_Parser/tptp_reconstruct_library.ML	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/TPTP/TPTP_Parser/tptp_reconstruct_library.ML	Thu Feb 15 12:11:00 2018 +0100
@@ -264,13 +264,13 @@
     | try_dest_All t = t
 
   val _ = @{assert}
-    ((@{term "! x. (! y. P) = True"}
+    ((@{term "\<forall>x. (\<forall>y. P) = True"}
       |> try_dest_All
       |> Term.strip_abs_vars)
      = [("x", @{typ "'a"})])
 
   val _ = @{assert}
-    ((@{prop "! x. (! y. P) = True"}
+    ((@{prop "\<forall>x. (\<forall>y. P) = True"}
       |> try_dest_All
       |> Term.strip_abs_vars)
      = [("x", @{typ "'a"})])
@@ -306,7 +306,7 @@
          Free ("x", @{typ "'a"})))
   in
     @{assert}
-      ((@{term "! x. All ((=) x)"}
+      ((@{term "\<forall>x. All ((=) x)"}
         |> strip_top_All_vars)
        = answer)
   end
@@ -642,7 +642,7 @@
      val simpset =
        empty_simpset ctxt
        |> Simplifier.add_simp
-           @{lemma "! x. P x & Q x \<equiv> (! x. P x) & (! x. Q x)"
+           @{lemma "\<forall>x. P x \<and> Q x \<equiv> (\<forall>x. P x) \<and> (\<forall>x. Q x)"
               by (rule eq_reflection, auto)}
    in
      CHANGED (asm_full_simp_tac simpset i)