aboutsummaryrefslogtreecommitdiff
path: root/proofs/clenvtac.mli
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2020-06-17 15:10:32 +0200
committerPierre-Marie Pédrot2020-06-24 15:38:24 +0200
commit34aeda3d701efd5dead8890588fb02bcdb4980d2 (patch)
tree9330fb20e4e7d95bac5d1550f4340bfed73efd67 /proofs/clenvtac.mli
parentb89584b989d8623a63e85b4a664a730d0f92ed65 (diff)
Merge Clenvtac into Clenv.
Having two different modules led to the availability of internal API in the mli.
Diffstat (limited to 'proofs/clenvtac.mli')
-rw-r--r--proofs/clenvtac.mli22
1 files changed, 0 insertions, 22 deletions
diff --git a/proofs/clenvtac.mli b/proofs/clenvtac.mli
deleted file mode 100644
index a34ec0e5be..0000000000
--- a/proofs/clenvtac.mli
+++ /dev/null
@@ -1,22 +0,0 @@
-(************************************************************************)
-(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * Copyright INRIA, CNRS and contributors *)
-(* <O___,, * (see version control and CREDITS file for authors & dates) *)
-(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(* * (see LICENSE file for the text of the license) *)
-(************************************************************************)
-
-(** Legacy components of the previous proof engine. *)
-
-open Clenv
-open EConstr
-open Unification
-
-(** Tactics *)
-val unify : ?flags:unify_flags -> constr -> unit Proofview.tactic
-val res_pf : ?with_evars:bool -> ?with_classes:bool -> ?flags:unify_flags -> clausenv -> unit Proofview.tactic
-
-val clenv_pose_dependent_evars : ?with_evars:bool -> clausenv -> clausenv
-val clenv_value_cast_meta : clausenv -> constr