lean2/tests/lean/run/goal.lean

5 lines
116 B
Text
Raw Normal View History

import standard
using tactic
theorem T {a b c d : Prop} (H : a) (H : b) (H : c) (H : d) : a
:= by state; assumption