lean2/tests/lean/run/premises.lean

10 lines
156 B
Text
Raw Normal View History

variable a : Prop
variables b c : Prop
premise Ha : a
premises (Hb : b) (Hc : c)
theorem tst : a ∧ b ∧ c :=
and.intro Ha (and.intro Hb Hc)
check tst