Skip to content

Commit 524d83d

Browse files
committed
workaround
1 parent 09e8dad commit 524d83d

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed

ProofWidgets/Component/Panel/Basic.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,8 @@
11
import ProofWidgets.Compat
22
import ProofWidgets.Component.Basic
33
import Lean.Elab.Tactic
4+
import Lean.Widget.Commands
5+
import Batteries.Tactic.OpenPrivate
46

57
namespace ProofWidgets
68
open Lean Elab Tactic
@@ -40,6 +42,8 @@ will show the geometry display alongside the usual tactic state throughout the p
4042
syntax (name := withPanelWidgetsTacticStx)
4143
"with_panel_widgets" "[" Widget.widgetInstanceSpec,+ "]" tacticSeq : tactic
4244

45+
open private Widget.elabWidgetInstanceSpec from Lean.Widget.Commands
46+
4347
@[tactic withPanelWidgetsTacticStx]
4448
def withPanelWidgets : Tactic
4549
| stx@`(tactic| with_panel_widgets [ $specs,* ] $seq) => do

0 commit comments

Comments
 (0)