aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@ens-lyon.fr>2017-09-01 16:02:01 +0200
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2018-07-03 13:39:18 +0200
commitd0b1ac17610bec74abaf122628b74c62643655d8 (patch)
treed10188301cb6b7a272cb64c5d9073b66b7d15264 /plugins
parent9ecaa34f6da55fda9743324d0f2212833e2e8487 (diff)
Coq_omega: remove unused Goal.enters
Diffstat (limited to 'plugins')
-rw-r--r--plugins/omega/coq_omega.ml10
1 files changed, 3 insertions, 7 deletions
diff --git a/plugins/omega/coq_omega.ml b/plugins/omega/coq_omega.ml
index 47eb043e6..e14c4e2ec 100644
--- a/plugins/omega/coq_omega.ml
+++ b/plugins/omega/coq_omega.ml
@@ -38,13 +38,9 @@ open OmegaSolver
(* Added by JCF, 09/03/98 *)
-let elim_id id =
- Proofview.Goal.enter begin fun gl ->
- simplest_elim (mkVar id)
- end
-let resolve_id id = Proofview.Goal.enter begin fun gl ->
- apply (mkVar id)
-end
+let elim_id id = simplest_elim (mkVar id)
+
+let resolve_id id = apply (mkVar id)
let display_time_flag = ref false
let display_system_flag = ref false