9 lines
224 B
Plaintext
9 lines
224 B
Plaintext
|
import LSpec
|
||
|
import Pantograph.Symbols
|
||
|
|
||
|
open Pantograph
|
||
|
|
||
|
def main := do
|
||
|
LSpec.lspecIO $
|
||
|
LSpec.test "Symbol parsing" (Lean.Name.str (.str (.str .anonymous "Lean") "Meta") "run" = Pantograph.str_to_name "Lean.Meta.run")
|