aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/omega
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2017-05-29 11:48:51 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2017-05-29 11:58:48 +0200
commitfd7f056b155b2ebaafa3251a3c136117ebefc3e3 (patch)
tree46ff14eb398806485d148757a2f34e1889ef7aaf /plugins/omega
parent4c1260299b707bd27765b0ab365092046b134a69 (diff)
Cleanup: removal of constr_of_global.
Constrintern.pf_global returns a global_reference, not a constr, adapt plugins accordingly, properly registering universes where necessary.
Diffstat (limited to 'plugins/omega')
-rw-r--r--plugins/omega/coq_omega.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/plugins/omega/coq_omega.ml b/plugins/omega/coq_omega.ml
index ee748567b..d7408e88e 100644
--- a/plugins/omega/coq_omega.ml
+++ b/plugins/omega/coq_omega.ml
@@ -39,10 +39,10 @@ open OmegaSolver
let elim_id id =
Proofview.Goal.enter { enter = begin fun gl ->
- simplest_elim (Tacmach.New.pf_global id gl)
+ simplest_elim (mkVar id)
end }
let resolve_id id = Proofview.Goal.enter { enter = begin fun gl ->
- apply (Tacmach.New.pf_global id gl)
+ apply (mkVar id)
end }
let timing timer_name f arg = f arg