2013-12-26 23:54:53 +00:00
|
|
|
(** import("tactic.lua") **)
|
2013-12-25 06:40:34 +00:00
|
|
|
Variables a b c : Bool
|
|
|
|
Axiom H : a \/ b
|
|
|
|
Theorem T (a b : Bool) : a \/ b => b \/ a.
|
|
|
|
apply Discharge.
|
|
|
|
apply (DisjCases H).
|
|
|
|
apply Disj2.
|
2013-12-26 23:54:53 +00:00
|
|
|
exact.
|
2013-12-25 06:40:34 +00:00
|
|
|
apply Disj1.
|
2013-12-26 23:54:53 +00:00
|
|
|
exact.
|
2013-12-25 06:40:34 +00:00
|
|
|
done.
|