aboutsummaryrefslogtreecommitdiff
path: root/proofs/logic.ml
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2019-04-05 02:30:45 +0200
committerEmilio Jesus Gallego Arias2019-04-05 15:05:53 +0200
commit54fdae0929f2a05a89cd5c463b9a739ab2e239b8 (patch)
tree80c38984687249bba8a66e24ad04a48de80c2bfa /proofs/logic.ml
parent3c06ce8dc3a95e5dfe3a4c0a9acdc7dd5dac75cb (diff)
[api] [proofs] Remove dependency of proofs on interp.
We perform some cleanup and remove dependency of `proofs/` on `interp/`, which seems logical. In fact, `interp` + `parsing` are quite self-contained, so if there is interest we could also make tactics to depend directly on proofs.
Diffstat (limited to 'proofs/logic.ml')
-rw-r--r--proofs/logic.ml1
1 files changed, 0 insertions, 1 deletions
diff --git a/proofs/logic.ml b/proofs/logic.ml
index 3581e90b79..a01ddf2388 100644
--- a/proofs/logic.ml
+++ b/proofs/logic.ml
@@ -63,7 +63,6 @@ let catchable_exception = function
| CErrors.UserError _ | TypeError _
| Proof.OpenProof _
(* abstract will call close_proof inside a tactic *)
- | Notation.PrimTokenNotationError _
| RefinerError _ | Indrec.RecursionSchemeError _
| Nametab.GlobalizationError _
(* reduction errors *)