Module Printer
These are the entry points for printing terms, context, tac, ...
val enable_unfocused_goal_printing : bool Stdlib.refval enable_goal_tags_printing : bool Stdlib.refval enable_goal_names_printing : bool Stdlib.ref
val pr_lconstr_env : Environ.env -> Evd.evar_map -> Constr.constr -> Pp.tval pr_lconstr_goal_style_env : Environ.env -> Evd.evar_map -> Constr.constr -> Pp.tval pr_constr_env : Environ.env -> Evd.evar_map -> Constr.constr -> Pp.tval pr_constr_goal_style_env : Environ.env -> Evd.evar_map -> Constr.constr -> Pp.tval pr_constr_n_env : Environ.env -> Evd.evar_map -> Notation_gram.tolerability -> Constr.constr -> Pp.t
val safe_pr_lconstr_env : Environ.env -> Evd.evar_map -> Constr.constr -> Pp.tval safe_pr_constr_env : Environ.env -> Evd.evar_map -> Constr.constr -> Pp.tval pr_econstr_env : Environ.env -> Evd.evar_map -> EConstr.t -> Pp.tval pr_leconstr_env : Environ.env -> Evd.evar_map -> EConstr.t -> Pp.tval pr_econstr_n_env : Environ.env -> Evd.evar_map -> Notation_gram.tolerability -> EConstr.t -> Pp.tval pr_etype_env : Environ.env -> Evd.evar_map -> EConstr.types -> Pp.tval pr_letype_env : Environ.env -> Evd.evar_map -> EConstr.types -> Pp.tval pr_open_constr_env : Environ.env -> Evd.evar_map -> Evd.open_constr -> Pp.tval pr_open_lconstr_env : Environ.env -> Evd.evar_map -> Evd.open_constr -> Pp.tval pr_constr_under_binders_env : Environ.env -> Evd.evar_map -> Ltac_pretype.constr_under_binders -> Pp.tval pr_lconstr_under_binders_env : Environ.env -> Evd.evar_map -> Ltac_pretype.constr_under_binders -> Pp.tval pr_goal_concl_style_env : Environ.env -> Evd.evar_map -> EConstr.types -> Pp.tval pr_ltype_env : Environ.env -> Evd.evar_map -> Constr.types -> Pp.tval pr_type_env : Environ.env -> Evd.evar_map -> Constr.types -> Pp.tval pr_closed_glob_n_env : Environ.env -> Evd.evar_map -> Notation_gram.tolerability -> Ltac_pretype.closed_glob_constr -> Pp.tval pr_closed_glob_env : Environ.env -> Evd.evar_map -> Ltac_pretype.closed_glob_constr -> Pp.tval pr_ljudge_env : Environ.env -> Evd.evar_map -> EConstr.unsafe_judgment -> Pp.t * Pp.tval pr_lglob_constr_env : Environ.env -> 'a Glob_term.glob_constr_g -> Pp.tval pr_glob_constr_env : Environ.env -> 'a Glob_term.glob_constr_g -> Pp.tval pr_lconstr_pattern_env : Environ.env -> Evd.evar_map -> Pattern.constr_pattern -> Pp.tval pr_constr_pattern_env : Environ.env -> Evd.evar_map -> Pattern.constr_pattern -> Pp.tval pr_cases_pattern : Glob_term.cases_pattern -> Pp.tval pr_sort : Evd.evar_map -> Sorts.t -> Pp.t
val pr_universe_instance : Evd.evar_map -> Univ.Instance.t -> Pp.tval pr_universe_instance_constraints : Evd.evar_map -> Univ.Instance.t -> Univ.Constraint.t -> Pp.tval pr_universe_ctx : Evd.evar_map -> ?variance:Univ.Variance.t array -> Univ.UContext.t -> Pp.tval pr_abstract_universe_ctx : Evd.evar_map -> ?variance:Univ.Variance.t array -> ?priv:Univ.ContextSet.t -> Univ.AUContext.t -> Pp.tval pr_universe_ctx_set : Evd.evar_map -> Univ.ContextSet.t -> Pp.tval pr_universes : Evd.evar_map -> ?variance:Univ.Variance.t array -> ?priv:Univ.ContextSet.t -> Declarations.universes -> Pp.t
val pr_global_env : Names.Id.Set.t -> Names.GlobRef.t -> Pp.tval pr_global : Names.GlobRef.t -> Pp.tval pr_constant : Environ.env -> Names.Constant.t -> Pp.tval pr_existential_key : Evd.evar_map -> Evar.t -> Pp.tval pr_existential : Environ.env -> Evd.evar_map -> Constr.existential -> Pp.tval pr_constructor : Environ.env -> Names.constructor -> Pp.tval pr_inductive : Environ.env -> Names.inductive -> Pp.tval pr_evaluable_reference : Names.evaluable_global_reference -> Pp.tval pr_pconstant : Environ.env -> Evd.evar_map -> Constr.pconstant -> Pp.tval pr_pinductive : Environ.env -> Evd.evar_map -> Constr.pinductive -> Pp.tval pr_pconstructor : Environ.env -> Evd.evar_map -> Constr.pconstructor -> Pp.t
val set_compact_context : bool -> unitDisplay compact contexts of goals (simple hyps on the same line)
val get_compact_context : unit -> boolval pr_context_unlimited : Environ.env -> Evd.evar_map -> Pp.tval pr_ne_context_of : Pp.t -> Environ.env -> Evd.evar_map -> Pp.tval pr_named_decl : Environ.env -> Evd.evar_map -> Constr.named_declaration -> Pp.tval pr_compacted_decl : Environ.env -> Evd.evar_map -> Constr.compacted_declaration -> Pp.tval pr_rel_decl : Environ.env -> Evd.evar_map -> Constr.rel_declaration -> Pp.tval pr_named_context : Environ.env -> Evd.evar_map -> Constr.named_context -> Pp.tval pr_named_context_of : Environ.env -> Evd.evar_map -> Pp.tval pr_rel_context : Environ.env -> Evd.evar_map -> Constr.rel_context -> Pp.tval pr_rel_context_of : Environ.env -> Evd.evar_map -> Pp.tval pr_context_of : Environ.env -> Evd.evar_map -> Pp.t
val pr_predicate : ('a -> Pp.t) -> (bool * 'a list) -> Pp.tval pr_cpred : Names.Cpred.t -> Pp.tval pr_idpred : Names.Id.Pred.t -> Pp.tval pr_transparent_state : TransparentState.t -> Pp.t
val pr_goal : ?diffs:bool -> ?og_s:Goal.goal Evd.sigma -> Goal.goal Evd.sigma -> Pp.tpr_goal ~diffs ~og_s g_sprints the goal specified byg_s. Ifdiffsis true, highlight the differences between the old goal,og_s, andg_s.g_sandog_sare records containing the goal and sigma for, respectively, the new and old proof steps, e.g.{ it = g ; sigma = sigma }.
val pr_subgoals : ?pr_first:bool -> ?diffs:bool -> ?os_map:(Evd.evar_map * Goal.goal Evar.Map.t) -> Pp.t option -> Evd.evar_map -> seeds:Goal.goal list -> shelf:Goal.goal list -> stack:int list -> unfocused:Goal.goal list -> goals:Goal.goal list -> Pp.tpr_subgoals ~pr_first ~diffs ~os_map close_cmd sigma ~seeds ~shelf ~stack ~unfocused ~goalsprints the goals ingoalsfollowed by the goals inunfocusedin a compact form (typically only the conclusion). Ifpr_firstis true, print the first goal in full.close_cmdis printed afterwards verbatim.If
diffsis true, then highlight diffs relative toos_mapin the output for first goal.os_mapcontains sigma for the old proof step and the goal map created byProof_diffs.make_goal_map.This function prints only the focused goals unless the corresponding option
enable_unfocused_goal_printingis set.seedsis for printing dependent evars (mainly for emacs proof tree mode).shelfis from Proof.proof and is used to identify shelved goals in a message if there are no more subgoals but there are non-instantiated existential variables.stackis used to print summary info on unfocused goals.
val pr_subgoal : int -> Evd.evar_map -> Goal.goal list -> Pp.tval pr_concl : int -> ?diffs:bool -> ?og_s:Goal.goal Evd.sigma -> Evd.evar_map -> Goal.goal -> Pp.tpr_concl n ~diffs ~og_s sigma gprints the conclusion of the goalgusingsigma. The output is labelled "subgoaln". Ifdiffsis true, highlight the differences between the old conclusion,og_s, andg+sigma.og_sis a record containing the old goal and sigma, e.g.{ it = g ; sigma = sigma }.
val pr_open_subgoals_diff : ?quiet:bool -> ?diffs:bool -> ?oproof:Proof.t -> Proof.t -> Pp.tpr_open_subgoals_diff ~quiet ~diffs ~oproof proofshows the context forproofas used by, for example, coqtop. The first active goal is printed with all its antecedents and the conclusion. The other active goals only show their conclusions. Ifdiffsis true, highlight the differences between the old proof,oproof, andproof.quietdisables printing messages as Feedback.
val pr_open_subgoals : proof:Proof.t -> Pp.tval pr_nth_open_subgoal : proof:Proof.t -> int -> Pp.tval pr_evar : Evd.evar_map -> (Evar.t * Evd.evar_info) -> Pp.tval pr_evars_int : Evd.evar_map -> shelf:Goal.goal list -> given_up:Goal.goal list -> int -> Evd.evar_info Evar.Map.t -> Pp.tval pr_evars : Evd.evar_map -> Evd.evar_info Evar.Map.t -> Pp.tval pr_ne_evar_set : Pp.t -> Pp.t -> Evd.evar_map -> Evar.Set.t -> Pp.tval print_and_diff : Proof.t option -> Proof.t option -> unitval print_dependent_evars : Evar.t option -> Evd.evar_map -> Evar.t list -> Pp.t
type axiom=|Constant of Names.Constant.t|Positive of Names.MutInd.t|Guarded of Names.GlobRef.t|TemplatePolymorphic of Names.MutInd.t|TypeInType of Names.GlobRef.tDeclarations for the "Print Assumption" command
type context_object=|Variable of Names.Id.t|Axiom of axiom * (Names.Label.t * Constr.rel_context * Constr.types) list|Opaque of Names.Constant.t|Transparent of Names.Constant.t
module ContextObjectSet : Stdlib.Set.S with type ContextObjectSet.elt = context_objectmodule ContextObjectMap : CMap.ExtS with type key = context_object and module Set := ContextObjectSetval pr_assumptionset : Environ.env -> Evd.evar_map -> Constr.types ContextObjectMap.t -> Pp.tval pr_goal_by_id : proof:Proof.t -> Names.Id.t -> Pp.tval pr_goal_emacs : proof:Proof.t option -> int -> int -> Pp.tval pr_typing_flags : Declarations.typing_flags -> Pp.t