aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/coercion.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-07-16 16:08:00 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-07-16 16:08:00 +0000
commit9e7cf06884565e3db81f63555ae259dbddcfe89d (patch)
tree9cd34bb248840a8ba0df89af276e4e03274d4203 /pretyping/coercion.mli
parent5542b28bc21866daf10634120cbd731c2092bd92 (diff)
Suppression de Rawterm.loc, branchement sur Util.loc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5911 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/coercion.mli')
-rw-r--r--pretyping/coercion.mli5
1 files changed, 3 insertions, 2 deletions
diff --git a/pretyping/coercion.mli b/pretyping/coercion.mli
index 36c981172..3a82e7ae8 100644
--- a/pretyping/coercion.mli
+++ b/pretyping/coercion.mli
@@ -9,6 +9,7 @@
(*i $Id$ i*)
(*i*)
+open Util
open Evd
open Names
open Term
@@ -35,11 +36,11 @@ val inh_coerce_to_sort :
(* [inh_conv_coerce_to loc env isevars j t] coerces [j] to an object of type
[t]; i.e. it inserts a coercion into [j], if needed, in such a way [t] and
[j.uj_type] are convertible; it fails if no coercion is applicable *)
-val inh_conv_coerce_to : Rawterm.loc ->
+val inh_conv_coerce_to : loc ->
env -> evar_defs -> unsafe_judgment -> constr -> unsafe_judgment
(* [inh_pattern_coerce_to loc env isevars pat ind1 ind2] coerces the Cases
pattern [pat] typed in [ind1] into a pattern typed in [ind2];
raises [Not_found] if no coercion found *)
val inh_pattern_coerce_to :
- Rawterm.loc -> cases_pattern -> inductive -> inductive -> cases_pattern
+ loc -> cases_pattern -> inductive -> inductive -> cases_pattern