package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type ident_decl = Misctypes.lident * universe_decl_expr option
type name_decl = Misctypes.lname * universe_decl_expr option
type notation = string
type explicitation =
  1. | ExplByPos of int * Names.Id.t option
  2. | ExplByName of Names.Id.t
type binder_kind =
  1. | Default of Decl_kinds.binding_kind
  2. | Generalized of Decl_kinds.binding_kind * Decl_kinds.binding_kind * bool
type abstraction_kind =
  1. | AbsLambda
  2. | AbsPi
type proj_flag = int option
type sign = bool
type raw_natural_number = string
type prim_token =
  1. | Numeral of raw_natural_number * sign
  2. | String of string
type instance_expr = Misctypes.glob_level list
type cases_pattern_expr_r =
  1. | CPatAlias of cases_pattern_expr * Misctypes.lname
  2. | CPatCstr of Libnames.reference * cases_pattern_expr list option * cases_pattern_expr list
  3. | CPatAtom of Libnames.reference option
  4. | CPatOr of cases_pattern_expr list
  5. | CPatNotation of notation * cases_pattern_notation_substitution * cases_pattern_expr list
  6. | CPatPrim of prim_token
  7. | CPatRecord of (Libnames.reference * cases_pattern_expr) list
  8. | CPatDelimiters of string * cases_pattern_expr
  9. | CPatCast of cases_pattern_expr * constr_expr
and cases_pattern_expr = cases_pattern_expr_r CAst.t
and cases_pattern_notation_substitution = cases_pattern_expr list * cases_pattern_expr list list
and constr_expr_r =
  1. | CRef of Libnames.reference * instance_expr option
  2. | CFix of Misctypes.lident * fix_expr list
  3. | CCoFix of Misctypes.lident * cofix_expr list
  4. | CProdN of local_binder_expr list * constr_expr
  5. | CLambdaN of local_binder_expr list * constr_expr
  6. | CLetIn of Misctypes.lname * constr_expr * constr_expr option * constr_expr
  7. | CAppExpl of proj_flag * Libnames.reference * instance_expr option * constr_expr list
  8. | CApp of proj_flag * constr_expr * (constr_expr * explicitation CAst.t option) list
  9. | CRecord of (Libnames.reference * constr_expr) list
  10. | CCases of Constr.case_style * constr_expr option * case_expr list * branch_expr list
  11. | CLetTuple of Misctypes.lname list * Misctypes.lname option * constr_expr option * constr_expr * constr_expr
  12. | CIf of constr_expr * Misctypes.lname option * constr_expr option * constr_expr * constr_expr
  13. | CHole of Evar_kinds.t option * Misctypes.intro_pattern_naming_expr * Genarg.raw_generic_argument option
  14. | CPatVar of Misctypes.patvar
  15. | CEvar of Glob_term.existential_name * (Names.Id.t * constr_expr) list
  16. | CSort of Misctypes.glob_sort
  17. | CCast of constr_expr * constr_expr Misctypes.cast_type
  18. | CNotation of notation * constr_notation_substitution
  19. | CGeneralization of Decl_kinds.binding_kind * abstraction_kind option * constr_expr
  20. | CPrim of prim_token
  21. | CDelimiters of string * constr_expr
and constr_expr = constr_expr_r CAst.t
and case_expr = constr_expr * Misctypes.lname option * cases_pattern_expr option
and branch_expr = (cases_pattern_expr list list * constr_expr) CAst.t
and recursion_order_expr =
  1. | CStructRec
  2. | CWfRec of constr_expr
  3. | CMeasureRec of constr_expr * constr_expr option
and local_binder_expr =
  1. | CLocalAssum of Misctypes.lname list * binder_kind * constr_expr
  2. | CLocalDef of Misctypes.lname * constr_expr * constr_expr option
  3. | CLocalPattern of (cases_pattern_expr * constr_expr option) CAst.t
and constr_notation_substitution = constr_expr list * constr_expr list list * cases_pattern_expr list * local_binder_expr list list
type constr_pattern_expr = constr_expr
type with_declaration_ast =
  1. | CWith_Module of Names.Id.t list CAst.t * Libnames.qualid CAst.t
  2. | CWith_Definition of Names.Id.t list CAst.t * universe_decl_expr option * constr_expr
type module_ast_r =
  1. | CMident of Libnames.qualid
  2. | CMapply of module_ast * module_ast
  3. | CMwith of module_ast * with_declaration_ast
and module_ast = module_ast_r CAst.t
OCaml

Innovation. Community. Security.