package coq
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>
On This Page
Formal proof management system
Install
dune-project
Dependency
Authors
Maintainers
Sources
coq-8.15.1.tar.gz
sha256=513e953b7183d478acb75fd6e80e4dc32ac1a918cf4343ac31a859cfb4e9aad2
doc/ltac2_plugin/Ltac2_plugin/Tac2quote/index.html
Module Ltac2_plugin.Tac2quoteSource
Syntactic quoting of expressions.
Contrarily to Tac2ffi, which lives on the semantic level, this module manipulates pure syntax of Ltac2. Its main purpose is to write notations.
Source
val constructor :
?loc:Loc.t ->
Tac2expr.ltac_constructor ->
Tac2expr.raw_tacexpr list ->
Tac2expr.raw_tacexprSource
val of_pair :
('a -> Tac2expr.raw_tacexpr) ->
('b -> Tac2expr.raw_tacexpr) ->
('a * 'b) CAst.t ->
Tac2expr.raw_tacexprSource
val of_open_constr :
?delimiters:Names.Id.t list ->
Constrexpr.constr_expr ->
Tac2expr.raw_tacexprid ↦ 'Control.hyp @id'
id ↦ 'Control.refine (fun () => Control.hyp @id')
id ↦ 'Control.refine (fun () => Control.hyp @id')
Generic arguments
Source
val wit_ltac1 :
(Names.Id.t CAst.t list * Ltac_plugin.Tacexpr.raw_tactic_expr,
Names.Id.t list * Ltac_plugin.Tacexpr.glob_tactic_expr)
Tac2dyn.Arg.tagLtac1 AST quotation, seen as a 'tactic'. Its type is unit in Ltac2.
Source
val wit_ltac1val :
(Names.Id.t CAst.t list * Ltac_plugin.Tacexpr.raw_tactic_expr,
Names.Id.t list * Ltac_plugin.Tacexpr.glob_tactic_expr)
Tac2dyn.Arg.tagLtac1 AST quotation, seen as a value-returning expression, with type Ltac1.t.
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>
On This Page