diff options
| author | Pierre-Marie Pédrot | 2021-01-22 19:43:55 +0100 |
|---|---|---|
| committer | Pierre-Marie Pédrot | 2021-01-22 19:43:55 +0100 |
| commit | 5986422fe75d017f75a0223f348d264638c1e33c (patch) | |
| tree | e63232c3924793e1eaedb0192d8ce95cf69d0077 /tactics | |
| parent | 7d5618684ef17fbb34246f041b3426d42825b85a (diff) | |
| parent | 4fffbe45f42517fbe41fbcf4bf77bfa72fff2579 (diff) | |
Merge PR #13761: Remove convert_concl_no_check (deprecated in 8.11)
Reviewed-by: Zimmi48
Reviewed-by: ppedrot
Diffstat (limited to 'tactics')
| -rw-r--r-- | tactics/tactics.ml | 3 | ||||
| -rw-r--r-- | tactics/tactics.mli | 4 |
2 files changed, 0 insertions, 7 deletions
diff --git a/tactics/tactics.ml b/tactics/tactics.ml index c64f583428..cbf12ac22f 100644 --- a/tactics/tactics.ml +++ b/tactics/tactics.ml @@ -156,9 +156,6 @@ let convert_hyp ~check ~reorder d = end end -let convert_concl_no_check = convert_concl ~check:false -let convert_hyp_no_check = convert_hyp ~check:false ~reorder:false - let convert_gen pb x y = Proofview.Goal.enter begin fun gl -> match Tacmach.New.pf_apply (Reductionops.infer_conv ~pb) gl x y with diff --git a/tactics/tactics.mli b/tactics/tactics.mli index a6471be549..d93f3bc434 100644 --- a/tactics/tactics.mli +++ b/tactics/tactics.mli @@ -35,10 +35,6 @@ val is_quantified_hypothesis : Id.t -> Proofview.Goal.t -> bool val introduction : Id.t -> unit Proofview.tactic val convert_concl : check:bool -> types -> cast_kind -> unit Proofview.tactic val convert_hyp : check:bool -> reorder:bool -> named_declaration -> unit Proofview.tactic -val convert_concl_no_check : types -> cast_kind -> unit Proofview.tactic -[@@ocaml.deprecated "use [Tactics.convert_concl]"] -val convert_hyp_no_check : named_declaration -> unit Proofview.tactic -[@@ocaml.deprecated "use [Tactics.convert_hyp]"] val mutual_fix : Id.t -> int -> (Id.t * int * constr) list -> int -> unit Proofview.tactic val fix : Id.t -> int -> unit Proofview.tactic |
