package coq
Formal proof management system
Install
Dune Dependency
Authors
Maintainers
Sources
coq-8.14.1.tar.gz
sha256=3cbfc1e1a72b16d4744f5b64ede59586071e31d9c11c811a0372060727bfd9c3
doc/coq-core.vernac/Vernacextend/index.html
Module Vernacextend
Source
Vernacular Extension data
Source
type vernac_classification =
| VtStartProof of vernac_start
| VtSideff of vernac_sideff_type
| VtQed of vernac_qed_type
| VtProofStep of {
proof_block_detection : proof_block_name option;
}
| VtQuery
| VtProofMode of string
| VtMeta
a terminator
abstracting anonymously its result
open type of delimiters
Interpretation of extended vernac phrases.
Source
type typed_vernac =
| VtDefault of unit -> unit
| VtNoProof of unit -> unit
| VtCloseProof of lemma:Declare.Proof.t -> pm:Declare.OblState.t -> Declare.OblState.t
| VtOpenProof of unit -> Declare.Proof.t
| VtModifyProof of pstate:Declare.Proof.t -> Declare.Proof.t
| VtReadProofOpt of pstate:Declare.Proof.t option -> unit
| VtReadProof of pstate:Declare.Proof.t -> unit
| VtReadProgram of stack:Vernacstate.LemmaStack.t option -> pm:Declare.OblState.t -> unit
| VtModifyProgram of pm:Declare.OblState.t -> Declare.OblState.t
| VtDeclareProgram of pm:Declare.OblState.t -> Declare.Proof.t
| VtOpenProofProgram of pm:Declare.OblState.t -> Declare.OblState.t * Declare.Proof.t
VERNAC EXTEND
Source
type (_, _) ty_sig =
| TyNil : (vernac_command, vernac_classification) ty_sig
| TyTerminal : string * ('r, 's) ty_sig -> ('r, 's) ty_sig
| TyNonTerminal : ('a, 'b, 'c) Extend.ty_user_symbol * ('r, 's) ty_sig -> ('a -> 'r, 'a -> 's) ty_sig
Source
val vernac_extend :
command:string ->
?classifier:(string -> vernac_classification) ->
?entry:Vernacexpr.vernac_expr Pcoq.Entry.t ->
ty_ml list ->
unit
Wrapper to dynamically extend vernacular commands.
VERNAC ARGUMENT EXTEND
Source
type 'a argument_rule =
| Arg_alias of 'a Pcoq.Entry.t
(*This is used because CAMLP5 parser can be dumb about rule factorization, which sometimes requires two entries to be the same.
*)| Arg_rules of 'a Pcoq.Production.t list
(*There is a discrepancy here as we use directly extension rules and thus entries instead of ty_user_symbol and thus arguments as roots.
*)
Source
type 'a vernac_argument = {
arg_printer : Environ.env -> Evd.evar_map -> 'a -> Pp.t;
arg_parsing : 'a argument_rule;
}
Source
val vernac_argument_extend :
name:string ->
'a vernac_argument ->
('a, unit, unit) Genarg.genarg_type * 'a Pcoq.Entry.t
STM classifiers
Standard constant classifiers
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>
On This Page