package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type t = t -> t
type accumulator
type tag = int
type arity = int
type reloc_table = (tag * arity) array
type annot_sw = {
  1. asw_ind : Names.inductive;
  2. asw_ci : Constr.case_info;
  3. asw_reloc : reloc_table;
  4. asw_finite : bool;
  5. asw_prefix : string;
}
val eq_annot_sw : annot_sw -> annot_sw -> bool
val hash_annot_sw : annot_sw -> int
type sort_annot = string * int
type rec_pos = int array
val eq_rec_pos : rec_pos -> rec_pos -> bool
type atom =
  1. | Arel of int
  2. | Aconstant of Constr.pconstant
  3. | Aind of Constr.pinductive
  4. | Asort of Sorts.t
  5. | Avar of Names.Id.t
  6. | Acase of annot_sw * accumulator * t * t -> t
  7. | Afix of t array * t array * rec_pos * int
  8. | Acofix of t array * t array * int * t
  9. | Acofixe of t array * t array * int * t
  10. | Aprod of Names.Name.t * t * t -> t
  11. | Ameta of Constr.metavariable * t
  12. | Aevar of Evar.t * t array
  13. | Aproj of Names.inductive * int * accumulator
type symbol =
  1. | SymbValue of t
  2. | SymbSort of Sorts.t
  3. | SymbName of Names.Name.t
  4. | SymbConst of Names.Constant.t
  5. | SymbMatch of annot_sw
  6. | SymbInd of Names.inductive
  7. | SymbMeta of Constr.metavariable
  8. | SymbEvar of Evar.t
  9. | SymbLevel of Univ.Level.t
  10. | SymbProj of Names.inductive * int
type symbols = symbol array
val empty_symbols : symbols
val mk_accu : atom -> t
val mk_rel_accu : int -> t
val mk_rels_accu : int -> int -> t array
val mk_constant_accu : Names.Constant.t -> Univ.Level.t array -> t
val mk_ind_accu : Names.inductive -> Univ.Level.t array -> t
val mk_sort_accu : Sorts.t -> Univ.Level.t array -> t
val mk_var_accu : Names.Id.t -> t
val mk_sw_accu : annot_sw -> accumulator -> t -> t -> t
val mk_prod_accu : Names.Name.t -> t -> t -> t
val mk_fix_accu : rec_pos -> int -> t array -> t array -> t
val mk_cofix_accu : int -> t array -> t array -> t
val mk_meta_accu : Constr.metavariable -> t
val mk_evar_accu : Evar.t -> t array -> t
val mk_proj_accu : (Names.inductive * int) -> accumulator -> t
val upd_cofix : t -> t -> unit
val force_cofix : t -> t
val mk_const : tag -> t
val mk_block : tag -> t array -> t
val mk_bool : bool -> t
val mk_int : int -> t
val mk_uint : Uint63.t -> t
val mk_float : Float64.t -> t
val napply : t -> t array -> t
val dummy_value : unit -> t
val atom_of_accu : accumulator -> atom
val args_of_accu : accumulator -> t array
val accu_nargs : accumulator -> int
val cast_accu : t -> accumulator
type block
val block_size : block -> int
val block_field : block -> int -> t
val block_tag : block -> int
type kind_of_value =
  1. | Vaccu of accumulator
  2. | Vfun of t -> t
  3. | Vconst of int
  4. | Vint64 of int64
  5. | Vfloat64 of float
  6. | Varray of t Parray.t
  7. | Vblock of block
val kind_of_value : t -> kind_of_value
val str_encode : 'a -> string
val str_decode : string -> 'a
val val_to_int : t -> int
val is_int : t -> bool
val head0 : t -> t -> t
val tail0 : t -> t -> t
val add : t -> t -> t -> t
val sub : t -> t -> t -> t
val mul : t -> t -> t -> t
val div : t -> t -> t -> t
val rem : t -> t -> t -> t
val l_sr : t -> t -> t -> t
val l_sl : t -> t -> t -> t
val l_and : t -> t -> t -> t
val l_xor : t -> t -> t -> t
val l_or : t -> t -> t -> t
val addc : t -> t -> t -> t
val subc : t -> t -> t -> t
val addCarryC : t -> t -> t -> t
val subCarryC : t -> t -> t -> t
val mulc : t -> t -> t -> t
val diveucl : t -> t -> t -> t
val div21 : t -> t -> t -> t -> t
val addMulDiv : t -> t -> t -> t -> t
val eq : t -> t -> t -> t
val lt : t -> t -> t -> t
val le : t -> t -> t -> t
val compare : t -> t -> t -> t
val print : t -> t
val no_check_head0 : t -> t
val no_check_tail0 : t -> t
val no_check_add : t -> t -> t
val no_check_sub : t -> t -> t
val no_check_mul : t -> t -> t
val no_check_div : t -> t -> t
val no_check_rem : t -> t -> t
val no_check_l_sr : t -> t -> t
val no_check_l_sl : t -> t -> t
val no_check_l_and : t -> t -> t
val no_check_l_xor : t -> t -> t
val no_check_l_or : t -> t -> t
val no_check_addc : t -> t -> t
val no_check_subc : t -> t -> t
val no_check_addCarryC : t -> t -> t
val no_check_subCarryC : t -> t -> t
val no_check_mulc : t -> t -> t
val no_check_diveucl : t -> t -> t
val no_check_div21 : t -> t -> t -> t
val no_check_addMulDiv : t -> t -> t -> t
val no_check_eq : t -> t -> t
val no_check_lt : t -> t -> t
val no_check_le : t -> t -> t
val no_check_compare : t -> t -> t
val is_float : t -> bool
val fopp : t -> t -> t
val fabs : t -> t -> t
val feq : t -> t -> t -> t
val flt : t -> t -> t -> t
val fle : t -> t -> t -> t
val fcompare : t -> t -> t -> t
val fclassify : t -> t -> t
val fadd : t -> t -> t -> t
val fsub : t -> t -> t -> t
val fmul : t -> t -> t -> t
val fdiv : t -> t -> t -> t
val fsqrt : t -> t -> t
val float_of_int : t -> t -> t
val normfr_mantissa : t -> t -> t
val frshiftexp : t -> t -> t
val ldshiftexp : t -> t -> t -> t
val next_up : t -> t -> t
val next_down : t -> t -> t
val no_check_fopp : t -> t
val no_check_fabs : t -> t
val no_check_feq : t -> t -> t
val no_check_flt : t -> t -> t
val no_check_fle : t -> t -> t
val no_check_fcompare : t -> t -> t
val no_check_fclassify : t -> t
val no_check_fadd : t -> t -> t
val no_check_fsub : t -> t -> t
val no_check_fmul : t -> t -> t
val no_check_fdiv : t -> t -> t
val no_check_fsqrt : t -> t
val no_check_float_of_int : t -> t
val no_check_normfr_mantissa : t -> t
val no_check_frshiftexp : t -> t
val no_check_ldshiftexp : t -> t -> t
val no_check_next_up : t -> t
val no_check_next_down : t -> t
val parray_of_array : t array -> t -> t
val is_parray : t -> bool
val arraymake : t -> t -> t -> t -> t
val arrayget : t -> t -> t -> t -> t
val arraydefault : t -> t -> t
val arrayset : t -> t -> t -> t -> t -> t
val arraycopy : t -> t -> t -> t
val arraylength : t -> t -> t -> t
val arrayinit : t -> t -> t -> t
val arraymap : t -> t -> t
val no_check_arraymake : t -> t -> t
val no_check_arrayget : t -> t -> t -> t
val no_check_arraydefault : t -> t
val no_check_arrayset : t -> t -> t -> t
val no_check_arraycopy : t -> t
val no_check_arraylength : t -> t