2013-12-26 15:54:53 -08:00
|
|
|
(** import("tactic.lua") **)
|
2013-12-24 22:40:34 -08: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 15:54:53 -08:00
|
|
|
exact.
|
2013-12-24 22:40:34 -08:00
|
|
|
apply Disj1.
|
2013-12-26 15:54:53 -08:00
|
|
|
exact.
|
2013-12-24 22:40:34 -08:00
|
|
|
done.
|