package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val __coq_plugin_name : string
type constr_expr_with_bindings = Constrexpr.constr_expr Tactypes.with_bindings
type glob_constr_with_bindings = Tacexpr.glob_constr_and_expr Tactypes.with_bindings
val pr_glob_constr_with_bindings_sign : 'a -> 'b -> 'c -> glob_constr_with_bindings_sign -> Pp.t
val pr_glob_constr_with_bindings : 'a -> 'b -> 'c -> glob_constr_with_bindings -> Pp.t
val pr_constr_expr_with_bindings : (Constrexpr.constr_expr -> 'a) -> 'b -> 'c -> constr_expr_with_bindings -> 'a
val interp_glob_constr_with_bindings : 'a -> Proof_type.goal Evd.sigma -> 'b -> Evd.evar_map * ('a * 'b)
val subst_strategy : 'a -> 'b -> 'b
val pr_strategy : 'a -> 'b -> 'c -> Rewrite.strategy -> Pp.t
val pr_raw_strategy : (Constrexpr.constr_expr -> Pp.t) -> (Constrexpr.constr_expr -> Pp.t) -> 'a -> raw_strategy -> Pp.t
val pr_glob_strategy : (Tacexpr.glob_constr_and_expr -> Pp.t) -> 'a -> 'b -> glob_strategy -> Pp.t
val rewstrategy : raw_strategy Pcoq.Entry.t
val db_strat : string -> ('a, 'b) Rewrite.strategy_ast
val cl_rewrite_clause_db : string -> Names.Id.t option -> unit Proofview.tactic
type binders_argtype = Constrexpr.local_binder_expr list
OCaml

Innovation. Community. Security.