aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--interp/syntax_def.mli1
-rw-r--r--pretyping/cases.mli1
-rw-r--r--pretyping/coercion.mli5
-rw-r--r--pretyping/detyping.mli1
-rw-r--r--pretyping/evarutil.mli3
-rw-r--r--pretyping/pretype_errors.mli1
-rw-r--r--pretyping/rawterm.ml2
-rw-r--r--pretyping/rawterm.mli2
8 files changed, 9 insertions, 7 deletions
diff --git a/interp/syntax_def.mli b/interp/syntax_def.mli
index 9083158ac..71b1d2991 100644
--- a/interp/syntax_def.mli
+++ b/interp/syntax_def.mli
@@ -9,6 +9,7 @@
(*i $Id$ i*)
(*i*)
+open Util
open Names
open Topconstr
open Rawterm
diff --git a/pretyping/cases.mli b/pretyping/cases.mli
index e05061f42..1985f7dd4 100644
--- a/pretyping/cases.mli
+++ b/pretyping/cases.mli
@@ -9,6 +9,7 @@
(*i $Id$ i*)
(*i*)
+open Util
open Names
open Term
open Evd
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
diff --git a/pretyping/detyping.mli b/pretyping/detyping.mli
index 7efaf4bbc..bf5c7bb56 100644
--- a/pretyping/detyping.mli
+++ b/pretyping/detyping.mli
@@ -9,6 +9,7 @@
(*i $Id$ i*)
(*i*)
+open Util
open Names
open Term
open Sign
diff --git a/pretyping/evarutil.mli b/pretyping/evarutil.mli
index 5e534f59c..2e0aa714d 100644
--- a/pretyping/evarutil.mli
+++ b/pretyping/evarutil.mli
@@ -9,6 +9,7 @@
(*i $Id$ i*)
(*i*)
+open Util
open Names
open Rawterm
open Term
@@ -93,7 +94,7 @@ val empty_valcon : val_constraint
val mk_valcon : constr -> val_constraint
val split_tycon :
- Rawterm.loc -> env -> evar_defs -> type_constraint ->
+ loc -> env -> evar_defs -> type_constraint ->
name * type_constraint * type_constraint
val valcon_of_tycon : type_constraint -> val_constraint
diff --git a/pretyping/pretype_errors.mli b/pretyping/pretype_errors.mli
index 4e98c8a2c..24eb04451 100644
--- a/pretyping/pretype_errors.mli
+++ b/pretyping/pretype_errors.mli
@@ -10,6 +10,7 @@
(*i*)
open Pp
+open Util
open Names
open Term
open Sign
diff --git a/pretyping/rawterm.ml b/pretyping/rawterm.ml
index 6e7f8f70f..555d608f1 100644
--- a/pretyping/rawterm.ml
+++ b/pretyping/rawterm.ml
@@ -19,8 +19,6 @@ open Nametab
(* Untyped intermediate terms, after ASTs and before constr. *)
-type loc = int * int
-
(* locs here refers to the ident's location, not whole pat *)
(* the last argument of PatCstr is a possible alias ident for the pattern *)
type cases_pattern =
diff --git a/pretyping/rawterm.mli b/pretyping/rawterm.mli
index e5b2a23fe..079fed34e 100644
--- a/pretyping/rawterm.mli
+++ b/pretyping/rawterm.mli
@@ -19,8 +19,6 @@ open Nametab
(* Untyped intermediate terms, after ASTs and before constr. *)
-type loc = int * int
-
(* locs here refers to the ident's location, not whole pat *)
(* the last argument of PatCstr is a possible alias ident for the pattern *)
type cases_pattern =