lean2/tests/lean/run/premises.lean
Leonardo de Moura 8ffadce4ab feat(frontends/lean): add "premise" and "premises" command
It is just an alternative notation for "variable" and "variables"

closes #429
2015-02-11 18:46:03 -08:00

9 lines
156 B
Text

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