aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/pfedit.ml
diff options
context:
space:
mode:
authorGravatar Arnaud Spiwack <arnaud@spiwack.net>2014-10-20 13:19:36 +0200
committerGravatar Arnaud Spiwack <arnaud@spiwack.net>2014-10-22 07:31:45 +0200
commit6074ee21f8c67830eb02f56c06fc94044e0ccfdf (patch)
treef35b9db68dbc75cdf4f0ddd0c941441db67dde33 /proofs/pfedit.ml
parent9f51aafebd5f3a00dabfe056772a300830b3c430 (diff)
Proofview: move [list_goto] to the [CList] module.
It is, after all, a generic function about lists.
Diffstat (limited to 'proofs/pfedit.ml')
-rw-r--r--proofs/pfedit.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index cb826bedc..b96a12c46 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -102,7 +102,7 @@ let solve ?with_end_tac gi tac pr =
Proof.run_tactic (Global.env ()) tac pr
with
| Proof_global.NoCurrentProof -> Errors.error "No focused proof"
- | Proofview.IndexOutOfRange ->
+ | CList.IndexOutOfRange ->
match gi with
| Vernacexpr.SelectNth i -> let msg = str "No such goal: " ++ int i ++ str "." in
Errors.errorlabstrm "" msg