aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/omega
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2018-07-05 12:56:27 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2018-07-05 12:56:27 +0200
commitd19605b7bfb8425b53be4cab30bef462c4fa4d14 (patch)
tree2bdcc15e217c24ca33b2fe48537c8632562a9ec1 /plugins/omega
parent7413f8532879c64e05ee0e8ca16693d74fe84ab9 (diff)
parent08b2fde7054a61e5468ef90eabb0d348730f170e (diff)
Merge PR #7746: Many small cleanups removing unused arguments and functions
Diffstat (limited to 'plugins/omega')
-rw-r--r--plugins/omega/coq_omega.ml10
1 files changed, 2 insertions, 8 deletions
diff --git a/plugins/omega/coq_omega.ml b/plugins/omega/coq_omega.ml
index 6f4138828..e14c4e2ec 100644
--- a/plugins/omega/coq_omega.ml
+++ b/plugins/omega/coq_omega.ml
@@ -38,15 +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 timing timer_name f arg = f arg
+let resolve_id id = apply (mkVar id)
let display_time_flag = ref false
let display_system_flag = ref false