aboutsummaryrefslogtreecommitdiff
path: root/checker/type_errors.mli
diff options
context:
space:
mode:
Diffstat (limited to 'checker/type_errors.mli')
-rw-r--r--checker/type_errors.mli106
1 files changed, 0 insertions, 106 deletions
diff --git a/checker/type_errors.mli b/checker/type_errors.mli
deleted file mode 100644
index 09703458ac..0000000000
--- a/checker/type_errors.mli
+++ /dev/null
@@ -1,106 +0,0 @@
-(************************************************************************)
-(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *)
-(* <O___,, * (see CREDITS file for the list of authors) *)
-(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(* * (see LICENSE file for the text of the license) *)
-(************************************************************************)
-
-(*i*)
-open Names
-open Cic
-open Environ
-(*i*)
-
-type unsafe_judgment = constr * constr
-
-(* Type errors. \label{typeerrors} *)
-
-(*i Rem: NotEnoughAbstractionInFixBody should only occur with "/i" Fix
- notation i*)
-type guard_error =
- (* Fixpoints *)
- | NotEnoughAbstractionInFixBody
- | RecursionNotOnInductiveType of constr
- | RecursionOnIllegalTerm of int * (env * constr) * int list * int list
- | NotEnoughArgumentsForFixCall of int
- (* CoFixpoints *)
- | CodomainNotInductiveType of constr
- | NestedRecursiveOccurrences
- | UnguardedRecursiveCall of constr
- | RecCallInTypeOfAbstraction of constr
- | RecCallInNonRecArgOfConstructor of constr
- | RecCallInTypeOfDef of constr
- | RecCallInCaseFun of constr
- | RecCallInCaseArg of constr
- | RecCallInCasePred of constr
- | NotGuardedForm of constr
- | ReturnPredicateNotCoInductive of constr
-
-type arity_error =
- | NonInformativeToInformative
- | StrongEliminationOnNonSmallType
- | WrongArity
-
-type type_error =
- | UnboundRel of int
- | UnboundVar of variable
- | NotAType of unsafe_judgment
- | BadAssumption of unsafe_judgment
- | ReferenceVariables of constr
- | ElimArity of pinductive * sorts_family list * constr * unsafe_judgment
- * (sorts_family * sorts_family * arity_error) option
- | CaseNotInductive of unsafe_judgment
- | WrongCaseInfo of inductive * case_info
- | NumberBranches of unsafe_judgment * int
- | IllFormedBranch of constr * int * constr * constr
- | Generalization of (Name.t * constr) * unsafe_judgment
- | ActualType of unsafe_judgment * constr
- | CantApplyBadType of
- (int * constr * constr) * unsafe_judgment * unsafe_judgment array
- | CantApplyNonFunctional of unsafe_judgment * unsafe_judgment array
- | IllFormedRecBody of guard_error * Name.t array * int
- | IllTypedRecBody of
- int * Name.t array * unsafe_judgment array * constr array
- | UnsatisfiedConstraints of Univ.constraints
-
-exception TypeError of env * type_error
-
-val error_unbound_rel : env -> int -> 'a
-
-val error_unbound_var : env -> variable -> 'a
-
-val error_not_type : env -> unsafe_judgment -> 'a
-
-val error_assumption : env -> unsafe_judgment -> 'a
-
-val error_reference_variables : env -> constr -> 'a
-
-val error_elim_arity :
- env -> pinductive -> sorts_family list -> constr -> unsafe_judgment ->
- (sorts_family * sorts_family * arity_error) option -> 'a
-
-val error_case_not_inductive : env -> unsafe_judgment -> 'a
-
-val error_number_branches : env -> unsafe_judgment -> int -> 'a
-
-val error_ill_formed_branch : env -> constr -> int -> constr -> constr -> 'a
-
-val error_actual_type : env -> unsafe_judgment -> constr -> 'a
-
-val error_cant_apply_not_functional :
- env -> unsafe_judgment -> unsafe_judgment array -> 'a
-
-val error_cant_apply_bad_type :
- env -> int * constr * constr ->
- unsafe_judgment -> unsafe_judgment array -> 'a
-
-val error_ill_formed_rec_body :
- env -> guard_error -> Name.t array -> int -> 'a
-
-val error_ill_typed_rec_body :
- env -> int -> Name.t array -> unsafe_judgment array -> constr array -> 'a
-
-val error_unsatisfied_constraints : env -> Univ.constraints -> 'a