Skip to content

Commit

Permalink
HolSmt: remove workaround for #1203
Browse files Browse the repository at this point in the history
Now that all known issues were fixed wrt. ARITH_PROVE not proving
goals that COOPER_PROVE could, we can remove this workaround, thus
making proof replay faster in some cases.
  • Loading branch information
someplaceguy authored and mn200 committed Apr 9, 2024
1 parent 70bec8c commit 84f2039
Showing 1 changed file with 1 addition and 6 deletions.
7 changes: 1 addition & 6 deletions src/HolSmt/Z3_ProofReplay.sml
Original file line number Diff line number Diff line change
Expand Up @@ -477,13 +477,8 @@ local
term that contains type real is provable by integer
arithmetic *)
profile "arith_prove(real)" RealField.REAL_ARITH_TAC goal
else (
else
profile "arith_prove(int)" intLib.ARITH_TAC goal
(* the following exception handler is a workaround for this issue:
https://github.com/HOL-Theorem-Prover/HOL/issues/1203 *)
handle Feedback.HOL_ERR _ =>
profile "arith_prove(cooper)" intLib.COOPER_TAC goal
)
val TRY = Tactical.TRY
val ap_tactic =
TRY AP_TERM_TAC >> TRY arith_tactic
Expand Down

0 comments on commit 84f2039

Please sign in to comment.