src/HOL/TPTP/TPTP_Proof_Reconstruction.thy
changeset 56245 84fc7dfa3cd4
parent 56220 4c43a2881b25
child 56252 b72e0a9d62b9
--- a/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy	Fri Mar 21 15:12:03 2014 +0100
+++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy	Fri Mar 21 20:33:56 2014 +0100
@@ -1670,7 +1670,7 @@
    (* @{const_name HOL.not_equal}, *)
    @{const_name HOL.False},
    @{const_name HOL.True},
-   @{const_name "==>"}]
+   @{const_name Pure.imp}]
 
 fun strip_qtfrs_tac ctxt =
   REPEAT_DETERM (HEADGOAL (rtac @{thm allI}))