368f9d347e
The previous approach was too fragile TODO: we should add separate parsing tables for tactics
10 lines
158 B
Text
10 lines
158 B
Text
import logic
|
|
open tactic
|
|
|
|
definition simple := apply _root_.trivial
|
|
|
|
tactic_hint simple
|
|
|
|
theorem foo : true
|
|
theorem foo2 (a : Prop) : a :
|
|
theorem foo3 : true
|