Open
Description
import Lean
syntax "foo " str : tactic
open Lean Elab
elab_rules : tactic
| `(foo $x:str) => logInfo x.getString
example : True := by
foo "hello" -- Error `tacticFoo_` has not been implemented
One has to write the elab_rules
above as
elab_rules : tactic
| `(tactic| foo $x:str) => logInfo x.getString