We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 09e8dad commit 524d83dCopy full SHA for 524d83d
ProofWidgets/Component/Panel/Basic.lean
@@ -1,6 +1,8 @@
1
import ProofWidgets.Compat
2
import ProofWidgets.Component.Basic
3
import Lean.Elab.Tactic
4
+import Lean.Widget.Commands
5
+import Batteries.Tactic.OpenPrivate
6
7
namespace ProofWidgets
8
open Lean Elab Tactic
@@ -40,6 +42,8 @@ will show the geometry display alongside the usual tactic state throughout the p
40
42
syntax (name := withPanelWidgetsTacticStx)
41
43
"with_panel_widgets" "[" Widget.widgetInstanceSpec,+ "]" tacticSeq : tactic
44
45
+open private Widget.elabWidgetInstanceSpec from Lean.Widget.Commands
46
+
47
@[tactic withPanelWidgetsTacticStx]
48
def withPanelWidgets : Tactic
49
| stx@`(tactic| with_panel_widgets [ $specs,* ] $seq) => do
0 commit comments