package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type recursion_scheme_error =
  1. | NotAllowedCaseAnalysis of bool * Term.sorts * Term.pinductive
  2. | NotMutualInScheme of Names.inductive * Names.inductive
  3. | NotAllowedDependentAnalysis of bool * Names.inductive
exception RecursionSchemeError of recursion_scheme_error
type dep_flag = bool
val build_case_analysis_scheme : Environ.env -> Evd.evar_map -> Term.pinductive -> dep_flag -> Term.sorts_family -> Evd.evar_map * Constr.t
val build_case_analysis_scheme_default : Environ.env -> Evd.evar_map -> Term.pinductive -> Term.sorts_family -> Evd.evar_map * Constr.t
val build_mutual_induction_scheme : Environ.env -> Evd.evar_map -> (Term.pinductive * dep_flag * Term.sorts_family) list -> Evd.evar_map * Term.constr list
val weaken_sort_scheme : Environ.env -> Evd.evar_map -> bool -> Term.sorts -> int -> Term.constr -> Term.types -> Evd.evar_map * Term.types * Term.constr
val elimination_suffix : Term.sorts_family -> string
val make_elimination_ident : Names.Id.t -> Term.sorts_family -> Names.Id.t
val case_suffix : string
OCaml

Innovation. Community. Security.