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