2014-10-28 00:12:25 +00:00
|
|
|
import logic
|
|
|
|
|
|
|
|
theorem tst1 (a b c : Prop) : a → b → a ∧ b :=
|
|
|
|
begin
|
|
|
|
intros,
|
|
|
|
apply and.intro,
|
2015-05-03 00:32:03 +00:00
|
|
|
repeat assumption
|
2014-10-28 00:12:25 +00:00
|
|
|
end
|
|
|
|
|
|
|
|
theorem tst2 (a b c : Prop) : a → b → a ∧ b :=
|
2015-05-03 00:32:03 +00:00
|
|
|
by intros; apply and.intro; repeat assumption
|