-
Notifications
You must be signed in to change notification settings - Fork 62
Open
Description
It is possible to make clauses using section variables survive the end of the section, contrary to what is stated in the documentation of coq.elpi.accumulate
.
From elpi Require Import elpi.
Elpi Command cmd.
Elpi Db db lp:{{
pred db? o:term.
}}.
Elpi Accumulate Db db.
#[synterp]
Elpi Accumulate cmd lp:{{
main _ :-
coq.env.begin-section "Dummy",
coq.env.end-section.
}}.
Elpi Accumulate cmd lp:{{
main _ :-
coq.env.begin-section "Dummy",
coq.env.add-section-variable "T" _ {{ Type }} T,
coq.elpi.accumulate _ "db" (clause _ _ (db? (global (const T)))),
coq.env.end-section.
}}.
Elpi cmd.
Section Dummy.
Variable (T U : Type).
Elpi Query cmd lp:{{
db? {{ T }}.
}}.
Fail Elpi Query cmd lp:{{
db? {{ U }}.
}}.
End Dummy.
Metadata
Metadata
Assignees
Labels
No labels