From 922ad0c1cb4a4badf4c9c2cd098285a008495519 Mon Sep 17 00:00:00 2001 From: Pierre-Marie Pédrot Date: Fri, 24 Jun 2016 14:54:42 +0200 Subject: Removing tactic compatibility layers in setoid_ring. --- plugins/setoid_ring/g_newring.ml4 | 6 +++--- plugins/setoid_ring/newring.ml | 7 +++---- plugins/setoid_ring/newring.mli | 6 +++--- 3 files changed, 9 insertions(+), 10 deletions(-) (limited to 'plugins/setoid_ring') diff --git a/plugins/setoid_ring/g_newring.ml4 b/plugins/setoid_ring/g_newring.ml4 index 767cf7ab7..216eb8b37 100644 --- a/plugins/setoid_ring/g_newring.ml4 +++ b/plugins/setoid_ring/g_newring.ml4 @@ -23,14 +23,14 @@ DECLARE PLUGIN "newring_plugin" TACTIC EXTEND protect_fv [ "protect_fv" string(map) "in" ident(id) ] -> - [ Proofview.V82.tactic (protect_tac_in map id) ] + [ protect_tac_in map id ] | [ "protect_fv" string(map) ] -> - [ Proofview.V82.tactic (protect_tac map) ] + [ protect_tac map ] END TACTIC EXTEND closed_term [ "closed_term" constr(t) "[" ne_reference_list(l) "]" ] -> - [ Proofview.V82.tactic (closed_term t l) ] + [ closed_term t l ] END open Pptactic diff --git a/plugins/setoid_ring/newring.ml b/plugins/setoid_ring/newring.ml index 57ef92032..55241ab2b 100644 --- a/plugins/setoid_ring/newring.ml +++ b/plugins/setoid_ring/newring.ml @@ -86,10 +86,10 @@ let protect_red map env sigma c = (mk_clos_but (lookup_map map c) (Esubst.subs_id 0) c);; let protect_tac map = - Proofview.V82.of_tactic (Tactics.reduct_option (protect_red map,DEFAULTcast) None);; + Tactics.reduct_option (protect_red map,DEFAULTcast) None let protect_tac_in map id = - Proofview.V82.of_tactic (Tactics.reduct_option (protect_red map,DEFAULTcast) (Some(id, Locus.InHyp)));; + Tactics.reduct_option (protect_red map,DEFAULTcast) (Some(id, Locus.InHyp)) (****************************************************************************) @@ -98,8 +98,7 @@ let closed_term t l = let open Quote_plugin in let l = List.map Universes.constr_of_global l in let cs = List.fold_right Quote.ConstrSet.add l Quote.ConstrSet.empty in - if Quote.closed_under cs t then tclIDTAC else tclFAIL 0 (mt()) -;; + if Quote.closed_under cs t then Proofview.tclUNIT () else Tacticals.New.tclFAIL 0 (mt()) (* TACTIC EXTEND echo | [ "echo" constr(t) ] -> diff --git a/plugins/setoid_ring/newring.mli b/plugins/setoid_ring/newring.mli index ca6aba9a0..f417c87cd 100644 --- a/plugins/setoid_ring/newring.mli +++ b/plugins/setoid_ring/newring.mli @@ -15,11 +15,11 @@ open Tacexpr open Proof_type open Newring_ast -val protect_tac_in : string -> Id.t -> tactic +val protect_tac_in : string -> Id.t -> unit Proofview.tactic -val protect_tac : string -> tactic +val protect_tac : string -> unit Proofview.tactic -val closed_term : constr -> global_reference list -> tactic +val closed_term : constr -> global_reference list -> unit Proofview.tactic val process_ring_mods : constr_expr ring_mod list -> -- cgit v1.2.3