aboutsummaryrefslogtreecommitdiff
path: root/kernel/type_errors.mli
diff options
context:
space:
mode:
authorherbelin2001-03-11 21:30:04 +0000
committerherbelin2001-03-11 21:30:04 +0000
commit3aa0e70a974c0b35801b42f8879c96c3188d98cf (patch)
tree96eec81ec2ff22271451cf10f1bd978b888d97d8 /kernel/type_errors.mli
parentc0754e3ae4f63466dd1b5ed535018bcc69bbaa5d (diff)
Déplacement des erreurs non noyau dans Pretype_errors ou Cases; localisation
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1445 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/type_errors.mli')
-rw-r--r--kernel/type_errors.mli22
1 files changed, 0 insertions, 22 deletions
diff --git a/kernel/type_errors.mli b/kernel/type_errors.mli
index e7e850c714..c45fac7218 100644
--- a/kernel/type_errors.mli
+++ b/kernel/type_errors.mli
@@ -49,20 +49,6 @@ type type_error =
| IllFormedRecBody of guard_error * name list * int * constr array
| IllTypedRecBody of int * name list * unsafe_judgment array
* types array
- | NotInductive of constr
- | MLCase of string * constr * constr * constr * constr
- | CantFindCaseType of constr
- | OccurCheck of int * constr
- | NotClean of int * constr
- | VarNotFound of identifier
- | UnexpectedType of constr * constr
- | NotProduct of constr
- (* Pattern-matching errors *)
- | BadPattern of constructor * constr
- | BadConstructor of constructor * inductive
- | WrongNumargConstructor of constructor_path * int
- | WrongPredicateArity of constr * constr * constr
- | NeedsInversion of constr * constr
exception TypeError of path_kind * env * type_error
@@ -107,11 +93,3 @@ val error_ill_typed_rec_body :
path_kind -> env -> int -> name list -> unsafe_judgment array
-> types array -> 'b
-val error_not_inductive : path_kind -> env -> constr -> 'a
-
-val error_ml_case : path_kind -> env ->
- string -> constr -> constr -> constr -> constr -> 'a
-
-val error_unexpected_type : env -> actual:constr -> expected:constr -> 'a
-
-val error_not_product : env -> constr -> 'a