aboutsummaryrefslogtreecommitdiff
path: root/proofs/refiner.mli
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2020-06-26 11:52:17 +0200
committerPierre-Marie Pédrot2020-06-29 15:15:13 +0200
commitf499083e65ba629e0232fad3f3bbc7fe21d9da2f (patch)
tree68992832115f17ccf9f22f49e4313951c4ba6cf5 /proofs/refiner.mli
parenta039e78c821ba6a0da5d3364b98491707eab8add (diff)
Remove the deprecated functions from refiner, moving them to Tacticals.
Diffstat (limited to 'proofs/refiner.mli')
-rw-r--r--proofs/refiner.mli98
1 files changed, 0 insertions, 98 deletions
diff --git a/proofs/refiner.mli b/proofs/refiner.mli
index a3cbfb5d5d..0ea630fdbc 100644
--- a/proofs/refiner.mli
+++ b/proofs/refiner.mli
@@ -24,107 +24,9 @@ val pf_hyps : Goal.goal sigma -> named_context
val refiner : check:bool -> Constr.t -> unit Proofview.tactic
-(** {6 Tacticals. } *)
-
-(** [tclIDTAC] is the identity tactic without message printing*)
-val tclIDTAC : tactic
-[@@ocaml.deprecated "Use Tactical.New.tclIDTAC"]
-val tclIDTAC_MESSAGE : Pp.t -> tactic
-[@@ocaml.deprecated]
-
-(** [tclEVARS sigma] changes the current evar map *)
-val tclEVARS : evar_map -> tactic
-[@@ocaml.deprecated "Use Proofview.Unsafe.tclEVARS"]
-
-
-(** [tclTHEN tac1 tac2 gls] applies the tactic [tac1] to [gls] and applies
- [tac2] to every resulting subgoals *)
-val tclTHEN : tactic -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHEN"]
-
-(** [tclTHENLIST [t1;..;tn]] applies [t1] THEN [t2] ... THEN [tn]. More
- convenient than [tclTHEN] when [n] is large *)
-val tclTHENLIST : tactic list -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENLIST"]
-
-(** [tclMAP f [x1..xn]] builds [(f x1);(f x2);...(f xn)] *)
-val tclMAP : ('a -> tactic) -> 'a list -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclMAP"]
-
-(** [tclTHEN_i tac1 tac2 gls] applies the tactic [tac1] to [gls] and applies
- [(tac2 i)] to the [i]{^ th} resulting subgoal (starting from 1) *)
-val tclTHEN_i : tactic -> (int -> tactic) -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHEN_i"]
-
-(** [tclTHENLAST tac1 tac2 gls] applies the tactic [tac1] to [gls] and [tac2]
- to the last resulting subgoal (previously called [tclTHENL]) *)
-val tclTHENLAST : tactic -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENLAST"]
-
-(** [tclTHENFIRST tac1 tac2 gls] applies the tactic [tac1] to [gls] and [tac2]
- to the first resulting subgoal *)
-val tclTHENFIRST : tactic -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENFIRST"]
-
-(** [tclTHENS tac1 [|t1 ; ... ; tn|] gls] applies the tactic [tac1] to
- [gls] and applies [t1],..., [tn] to the [n] resulting subgoals. Raises
- an error if the number of resulting subgoals is not [n] *)
-val tclTHENSV : tactic -> tactic array -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENSV"]
-
-(** Same with a list of tactics *)
-val tclTHENS : tactic -> tactic list -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENS"]
-
-(** [tclTHENS3PARTS tac1 [|t1 ; ... ; tn|] tac2 [|t'1 ; ... ; t'm|] gls]
- applies the tactic [tac1] to [gls] then, applies [t1], ..., [tn] to
- the first [n] resulting subgoals, [t'1], ..., [t'm] to the last [m]
- subgoals and [tac2] to the rest of the subgoals in the middle. Raises an
- error if the number of resulting subgoals is strictly less than [n+m] *)
-val tclTHENS3PARTS : tactic -> tactic array -> tactic -> tactic array -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENS3PARTS"]
-
-(** [tclTHENSLASTn tac1 [t1 ; ... ; tn] tac2 gls] applies [t1],...,[tn] on the
- last [n] resulting subgoals and [tac2] on the remaining first subgoals *)
-val tclTHENSLASTn : tactic -> tactic -> tactic array -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENSLASTn"]
-
-(** [tclTHENSFIRSTn tac1 [t1 ; ... ; tn] tac2 gls] first applies [tac1], then
- applies [t1],...,[tn] on the first [n] resulting subgoals and
- [tac2] for the remaining last subgoals (previously called tclTHENST) *)
-val tclTHENSFIRSTn : tactic -> tactic array -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENSFIRSTn"]
-
(** A special exception for levels for the Fail tactic *)
exception FailError of int * Pp.t Lazy.t
(** Takes an exception and either raise it at the next
level or do nothing. *)
val catch_failerror : Exninfo.iexn -> unit
-
-val tclORELSE0 : tactic -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclORELSE0"]
-val tclORELSE : tactic -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclORELSE"]
-val tclREPEAT : tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclREPEAT"]
-val tclFIRST : tactic list -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclFIRST"]
-val tclTRY : tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTRY"]
-val tclTHENTRY : tactic -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclTHENTRY"]
-val tclCOMPLETE : tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclCOMPLETE"]
-val tclAT_LEAST_ONCE : tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclAT_LEAST_ONCE"]
-val tclFAIL : int -> Pp.t -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclFAIL"]
-val tclFAIL_lazy : int -> Pp.t Lazy.t -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclFAIL_lazy"]
-val tclDO : int -> tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclDO"]
-val tclPROGRESS : tactic -> tactic
-[@@ocaml.deprecated "Use Tactical.New.tclPROGRESS"]
-val tclSHOWHYPS : tactic -> tactic
-[@@ocaml.deprecated "Internal tactic. Do not use."]