From bda7852cb0896727389935f420eec0e8e3315cf7 Mon Sep 17 00:00:00 2001 From: Pierre-Marie Pédrot Date: Thu, 12 Jun 2014 15:04:06 +0200 Subject: Passing some tactics to the new monad type. --- plugins/fourier/fourierR.ml | 22 ++++++++++------------ 1 file changed, 10 insertions(+), 12 deletions(-) (limited to 'plugins/fourier') diff --git a/plugins/fourier/fourierR.ml b/plugins/fourier/fourierR.ml index d34d50364..1f6ece602 100644 --- a/plugins/fourier/fourierR.ml +++ b/plugins/fourier/fourierR.ml @@ -422,18 +422,16 @@ let my_cut c gl= let exact = exact_check;; -let tac_use h = match h.htype with - "Rlt" -> exact h.hname - |"Rle" -> exact h.hname - |"Rgt" -> (tclTHEN (apply (get coq_Rfourier_gt_to_lt)) - (exact h.hname)) - |"Rge" -> (tclTHEN (apply (get coq_Rfourier_ge_to_le)) - (exact h.hname)) - |"eqTLR" -> (tclTHEN (apply (get coq_Rfourier_eqLR_to_le)) - (exact h.hname)) - |"eqTRL" -> (tclTHEN (apply (get coq_Rfourier_eqRL_to_le)) - (exact h.hname)) - |_->assert false +let tac_use h = + let tac = Proofview.V82.of_tactic (exact h.hname) in + match h.htype with + "Rlt" -> tac + |"Rle" -> tac + |"Rgt" -> (tclTHEN (apply (get coq_Rfourier_gt_to_lt)) tac) + |"Rge" -> (tclTHEN (apply (get coq_Rfourier_ge_to_le)) tac) + |"eqTLR" -> (tclTHEN (apply (get coq_Rfourier_eqLR_to_le)) tac) + |"eqTRL" -> (tclTHEN (apply (get coq_Rfourier_eqRL_to_le)) tac) + |_->assert false ;; (* -- cgit v1.2.3