aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tacinterp.mli
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-12 21:08:00 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-12 21:08:00 +0000
commit62e5258743a296a59535c97f359a196ff7569188 (patch)
treee0e8761c6eff54e843516c7c15998cd927a69071 /tactics/tacinterp.mli
parent38c56b1988f07e4d21ec07c8de12ad63c82f9c1e (diff)
Moving coercion functions out of Tacinterp.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16577 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/tacinterp.mli')
-rw-r--r--tactics/tacinterp.mli4
1 files changed, 1 insertions, 3 deletions
diff --git a/tactics/tacinterp.mli b/tactics/tacinterp.mli
index 7c04899f3..8395306b6 100644
--- a/tactics/tacinterp.mli
+++ b/tactics/tacinterp.mli
@@ -21,7 +21,7 @@ open Misctypes
module Value :
sig
- type t
+ type t = tlevel generic_argument
val of_constr : constr -> t
val to_constr : t -> constr option
val of_int : int -> t
@@ -119,8 +119,6 @@ val declare_xml_printer :
(** Internals that can be useful for syntax extensions. *)
-exception CannotCoerceTo of string
-
val interp_ltac_var : (value -> 'a) -> interp_sign -> Environ.env option -> Id.t Loc.located -> 'a
val interp_int : interp_sign -> Id.t Loc.located -> int