2013-12-30 21:35:37 +00:00
|
|
|
Import tactic.
|
|
|
|
Import int.
|
2013-12-26 23:54:53 +00:00
|
|
|
|
2013-12-05 11:22:12 +00:00
|
|
|
Variable f : Int -> Int -> Bool
|
|
|
|
Variable P : Int -> Int -> Bool
|
|
|
|
Axiom Ax1 (x y : Int) (H : P x y) : (f x y)
|
|
|
|
Theorem T1 (a : Int) : (P a a) => (f a a).
|
2013-12-26 23:54:53 +00:00
|
|
|
apply Discharge.
|
|
|
|
apply Ax1.
|
|
|
|
exact.
|
|
|
|
done.
|
2013-12-05 11:22:12 +00:00
|
|
|
Variable b : Int
|
|
|
|
Axiom Ax2 (x : Int) : (f x b)
|
|
|
|
(**
|
2013-12-26 23:54:53 +00:00
|
|
|
simple_tac = Repeat(OrElse(imp_tac(), assumption_tac(), apply_tac("Ax2"), apply_tac("Ax1")))
|
2013-12-05 11:22:12 +00:00
|
|
|
**)
|
|
|
|
Theorem T2 (a : Int) : (P a a) => (f a a).
|
2013-12-26 23:54:53 +00:00
|
|
|
simple_tac.
|
|
|
|
done.
|
|
|
|
|
|
|
|
Theorem T3 (a : Int) : (P a a) => (f a a).
|
|
|
|
Repeat (OrElse (apply Discharge) exact (apply Ax2) (apply Ax1)).
|
|
|
|
done.
|
2013-12-05 11:22:12 +00:00
|
|
|
|
2013-12-26 23:54:53 +00:00
|
|
|
Show Environment 2.
|