You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
I get suggestions for things like SepExprFacts#env#heq_ST_heq_mor_Proper from theorems like
GlobalAddParametricMorphism : (SE.sexprD funcs preds U G) with
signature (SE.heq funcs preds U G cs ==> SE.ST.heq cs)
as heq_ST_heq_mor.
Proof.
unfold SE.heq; simpl; auto.
Qed.
and I get suggestions for things like imports#Straightline__subproof when I use [abstract] inside of [Defined]. In the latter case, [Set Suggest Proof Using] should make a suggestion for the transparent definition, or make no suggestion at all (if no [Proof using] directive would result in pushing the [abstract] to a worker). In the former case, [Set Suggest Proof Using] should probably make a suggestion for the name given in [as foo], but I'm not completely sure about this.
Note: the issue was created automatically with bugzilla2github tool
Original bug ID: BZ#4004
From: @JasonGross
Reported version: 8.5
CC: @gares
The text was updated successfully, but these errors were encountered: