package coq
Install
Dune Dependency
Authors
Maintainers
Sources
sha256=513e953b7183d478acb75fd6e80e4dc32ac1a918cf4343ac31a859cfb4e9aad2
doc/coq-core.printing/Proof_diffs/index.html
Module Proof_diffs
Source
Name of Diffs option
Returns true if the diffs option is "on" or "removed"
Returns true if the diffs option is "removed"
controls whether color output is enabled
true indicates that color output is enabled
val diff_goal_ide :
(Goal.goal * Evd.evar_map) option ->
Goal.goal ->
Evd.evar_map ->
Pp.t list * Pp.t
Computes the diff between the goals of two Proofs and returns the highlighted lists of hypotheses and conclusions.
If the strings used to display the goal are not lexable (this is believed unlikely), this routine will generate a Diff_Failure. This routine may also raise Diff_Failure under some "impossible" conditions.
If you want to make your call especially bulletproof, catch these exceptions, print a user-visible message, then recall this routine with the first argument set to None, which will skip the diff.
Computes the diff between two goals
If the strings used to display the goal are not lexable (this is believed unlikely), this routine will generate a Diff_Failure. This routine may also raise Diff_Failure under some "impossible" conditions.
If you want to make your call especially bulletproof, catch these exceptions, print a user-visible message, then recall this routine with the first argument set to None, which will skip the diff.
Convert a string to a list of token strings using the lexer
val pr_letype_env :
?lax:bool ->
?goal_concl_style:bool ->
Environ.env ->
Evd.evar_map ->
?impargs:Glob_term.binding_kind list ->
EConstr.types ->
Pp.t
val pr_leconstr_env :
?lax:bool ->
?inctx:bool ->
?scope:Notation_term.scope_name ->
Environ.env ->
Evd.evar_map ->
EConstr.constr ->
Pp.t
val pr_lconstr_env :
?lax:bool ->
?inctx:bool ->
?scope:Notation_term.scope_name ->
Environ.env ->
Evd.evar_map ->
Constr.constr ->
Pp.t
Computes diffs for a single conclusion
Generates a map from np
to op
that maps changed goals to their prior forms. The map doesn't include entries for unchanged goals; unchanged goals will have the same goal id in both versions.
op
and np
must be from the same proof document and op
must be for a state before np
.
val diff_hyps :
string list list ->
hyp_info CString.Map.t ->
string list list ->
hyp_info CString.Map.t ->
Pp.t list