package coq
Install
Dune Dependency
Authors
Maintainers
Sources
sha256=73466e61f229b23b4daffdd964be72bd7a110963b9d84bd4a86bb05c5dc19ef3
doc/coq-core.interp/Constrexpr_ops/index.html
Module Constrexpr_ops
Source
Constrexpr_ops: utilities on constr_expr
Equalities on constr_expr
related types
Equality on explicitation
.
val constr_expr_eq_gen :
(Constrexpr.constr_expr -> Constrexpr.constr_expr -> bool) ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr ->
bool
Equality on constr_expr
. This is a syntactical one, which is oblivious to some parsing details, including locations.
Equality on local_binder_expr
. Same properties as constr_expr_eq
.
Equality on binder_kind
Retrieving locations
Constructors
Term constructors
Basic form of the corresponding constructors
val mkCastC :
(Constrexpr.constr_expr * Constr.cast_kind * Constrexpr.constr_expr) ->
Constrexpr.constr_expr
val mkLambdaC :
(Names.lname list
* Constrexpr.binder_kind
* Constrexpr.constr_expr
* Constrexpr.constr_expr) ->
Constrexpr.constr_expr
val mkLetInC :
(Names.lname
* Constrexpr.constr_expr
* Constrexpr.constr_expr option
* Constrexpr.constr_expr) ->
Constrexpr.constr_expr
val mkProdC :
(Names.lname list
* Constrexpr.binder_kind
* Constrexpr.constr_expr
* Constrexpr.constr_expr) ->
Constrexpr.constr_expr
Basic form of application, collapsing nested applications
Optimized constructors: does not add a constructor for an empty binder list
val mkLambdaCN :
?loc:Loc.t ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr
val mkProdCN :
?loc:Loc.t ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr
Aliases for the corresponding constructors; generally mkLambdaCN
and mkProdCN
should be preferred
val mkCLambdaN :
?loc:Loc.t ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr
val mkCProdN :
?loc:Loc.t ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr
Pattern constructors
val mkCPatOr :
?loc:Loc.t ->
Constrexpr.cases_pattern_expr list ->
Constrexpr.cases_pattern_expr
Interpretation of a list of patterns as a disjunctive pattern (optimized)
val mkAppPattern :
?loc:Loc.t ->
Constrexpr.cases_pattern_expr ->
Constrexpr.cases_pattern_expr list ->
Constrexpr.cases_pattern_expr
Apply a list of pattern arguments to a pattern
Destructors
FIXME: nothing to do here
Destruct terms of the form CRef (Ident _)
.
Destruct terms of the form CRef (Ident _)
or CHole _
.
Binder manipulation
Retrieve a list of binding names from a list of binders.
Same as names_of_local_binder_exprs
, but does not take the let
bindings into account.
Folds and maps
val fold_constr_expr_with_binders :
(Names.Id.t -> 'a -> 'a) ->
('a -> 'b -> Constrexpr.constr_expr -> 'b) ->
'a ->
'b ->
Constrexpr.constr_expr ->
'b
Used in typeclasses
Used in correctness and interface; absence of var capture not guaranteed in pattern-matching clauses and in binders of the form x,y:T(x)
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
val replace_vars_constr_expr :
Names.Id.t Names.Id.Map.t ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr
Return all (non-qualified) names treating binders as names
val split_at_annot :
Constrexpr.local_binder_expr list ->
Names.lident option ->
Constrexpr.local_binder_expr list * Constrexpr.local_binder_expr list
val ntn_loc :
?loc:Loc.t ->
Constrexpr.constr_notation_substitution ->
Constrexpr.notation ->
(int * int) list
val patntn_loc :
?loc:Loc.t ->
Constrexpr.cases_pattern_notation_substitution ->
Constrexpr.notation ->
(int * int) list