aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/pretype_errors.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-06-27 21:37:56 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-06-28 18:52:55 +0200
commit1f0e44c96872196d0051618de77c4735eb447540 (patch)
tree8b69aa789ebff430d021af431ad9ad453883ba25 /pretyping/pretype_errors.mli
parentefa921c807e48cfc19943d2bfd7f4eb11f8f9e09 (diff)
Moved code for finding subterms (pattern, induction, set, generalize, ...)
into a specific new cleaned file find_subterm.ml. This makes things clearer but also solves some dependencies problem between Evd, Termops and Pretype_errors.
Diffstat (limited to 'pretyping/pretype_errors.mli')
-rw-r--r--pretyping/pretype_errors.mli6
1 files changed, 5 insertions, 1 deletions
diff --git a/pretyping/pretype_errors.mli b/pretyping/pretype_errors.mli
index f8e39f316..e816463e7 100644
--- a/pretyping/pretype_errors.mli
+++ b/pretyping/pretype_errors.mli
@@ -24,6 +24,10 @@ type unification_error =
| InstanceNotSameType of existential_key * env * types * types
| UnifUnivInconsistency of Univ.univ_inconsistency
+type position =(Id.t * Locus.hyp_location_flag) option
+
+type subterm_unification_error = bool * (position * int * constr) * (position * int * constr) * (constr * constr * unification_error) option
+
type pretype_error =
(** Old Case *)
| CantFindCaseType of constr
@@ -47,7 +51,7 @@ type pretype_error =
| UnexpectedType of constr * constr
| NotProduct of constr
| TypingError of type_error
- | CannotUnifyOccurrences of Termops.subterm_unification_error
+ | CannotUnifyOccurrences of subterm_unification_error
exception PretypeError of env * Evd.evar_map * pretype_error