5 lines
116 B
Text
5 lines
116 B
Text
|
import standard
|
||
|
using tactic
|
||
|
|
||
|
theorem T {a b c d : Prop} (H : a) (H : b) (H : c) (H : d) : a
|
||
|
:= by state; assumption
|