8ffadce4ab
It is just an alternative notation for "variable" and "variables" closes #429
9 lines
156 B
Text
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
|