diff -r f14f17e656a6 -r 9e2a65912111 src/HOL/TPTP/TPTP_Interpret_Test.thy --- a/src/HOL/TPTP/TPTP_Interpret_Test.thy Thu Mar 03 14:03:06 2016 +0100 +++ b/src/HOL/TPTP/TPTP_Interpret_Test.thy Thu Mar 03 15:23:02 2016 +0100 @@ -129,7 +129,7 @@ val t1 = (parse_timed file |> fst) val t2 = (interpret_timed timeout file thy |> fst) handle exn => (*FIXME*) - if Exn.is_interrupt exn then reraise exn + if Exn.is_interrupt exn then Exn.reraise exn else (warning (" test: file " ^ Path.print file ^ " raised exception: " ^ Runtime.exn_message exn);