2014-07-02 20:14:50 +00:00
|
|
|
import standard
|
|
|
|
using tactic
|
2014-06-30 01:26:07 +00:00
|
|
|
|
|
|
|
theorem tst {A B : Bool} (H1 : A) (H2 : B) : A ∧ B ∧ A
|
2014-07-03 01:10:42 +00:00
|
|
|
:= by apply and_intro; state; assumption; apply and_intro; !assumption
|
2014-07-02 20:14:50 +00:00
|
|
|
check tst
|
|
|
|
|
|
|
|
theorem tst2 {A B : Bool} (H1 : A) (H2 : B) : A ∧ B ∧ A
|
2014-07-03 01:10:42 +00:00
|
|
|
:= by !((apply @and_intro | assumption) ; trace "STEP"; state; trace "----------")
|
2014-07-02 20:14:50 +00:00
|
|
|
|
|
|
|
check tst2
|
|
|
|
|