aboutsummaryrefslogtreecommitdiff
path: root/ide
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-05-25 16:43:01 +0200
committerEmilio Jesus Gallego Arias2020-06-26 14:38:11 +0200
commit030bb57d4b7e70d45379cab61903b75bf7a41b19 (patch)
treed69b91d1210cb129626a8deeaca6a2d1bf6fad39 /ide
parentb143d124e140628e5974da4af1b8a70a4d534598 (diff)
[declare] Reify Proof.t API into the Proof module.
This is in preparation for the next commit which will clean-up the current API flow in `Declare`.
Diffstat (limited to 'ide')
-rw-r--r--ide/coqide/idetop.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/ide/coqide/idetop.ml b/ide/coqide/idetop.ml
index bd99cbed1b..2adc35ae3e 100644
--- a/ide/coqide/idetop.ml
+++ b/ide/coqide/idetop.ml
@@ -343,7 +343,7 @@ let search flags =
let pstate = Vernacstate.Declare.get_pstate () in
let sigma, env = match pstate with
| None -> let env = Global.env () in Evd.(from_env env, env)
- | Some p -> Declare.get_goal_context p 1 in
+ | Some p -> Declare.Proof.get_goal_context p 1 in
List.map export_coq_object (Search.interface_search env sigma (
List.map (fun (c, b) -> (import_search_constraint c, b)) flags)
)