package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val asymmetric_patterns : bool Pervasives.ref
  • deprecated use Constrexpr_ops.asymmetric_patterns
  • deprecated use Constrexpr_ops.split_at_annot
val ntn_loc : ?loc:Loc.t -> Constrexpr.constr_notation_substitution -> string -> (int * int) list
  • deprecated use Constrexpr_ops.ntn_loc
val patntn_loc : ?loc:Loc.t -> Constrexpr.cases_pattern_notation_substitution -> string -> (int * int) list
  • deprecated use Constrexpr_ops.patntn_loc
val error_invalid_pattern_notation : ?loc:Loc.t -> unit -> 'a
  • deprecated use Constrexpr_ops.error_invalid_pattern_notation
  • deprecated use Constrexpr_ops.free_vars_of_constr_expr
val free_vars_of_constr_expr : Constrexpr.constr_expr -> Names.Id.Set.t
  • deprecated use Constrexpr_ops.free_vars_of_constr_expr
val occur_var_constr_expr : Names.Id.t -> Constrexpr.constr_expr -> bool
  • deprecated use Constrexpr_ops.occur_var_constr_expr
val ids_of_cases_indtype : Constrexpr.cases_pattern_expr -> Names.Id.Set.t
  • deprecated use Constrexpr_ops.ids_of_cases_indtype
val fold_constr_expr_with_binders : (Names.Id.t -> 'a -> 'a) -> ('a -> 'b -> Constrexpr.constr_expr -> 'b) -> 'a -> 'b -> Constrexpr.constr_expr -> 'b
  • deprecated use Constrexpr_ops.fold_constr_expr_with_binders
val map_constr_expr_with_binders : (Names.Id.t -> 'a -> 'a) -> ('a -> Constrexpr.constr_expr -> Constrexpr.constr_expr) -> 'a -> Constrexpr.constr_expr -> Constrexpr.constr_expr
  • deprecated use Constrexpr_ops.map_constr_expr_with_binders
OCaml

Innovation. Community. Security.