2014-01-01 21:52:25 +00:00
|
|
|
Import Int
|
2013-12-28 20:04:56 +00:00
|
|
|
Import tactic
|
2013-12-23 01:11:36 +00:00
|
|
|
SetOption pp::implicit true
|
2013-12-23 01:57:51 +00:00
|
|
|
SetOption pp::coercion true
|
|
|
|
SetOption pp::notation false
|
2013-12-22 22:10:42 +00:00
|
|
|
Variable vector (A : Type) (sz : Nat) : Type
|
|
|
|
Variable read {A : Type} {sz : Nat} (v : vector A sz) (i : Nat) (H : i < sz) : A
|
|
|
|
Variable V1 : vector Int 10
|
2013-12-26 23:54:53 +00:00
|
|
|
Definition D := read V1 1 (by trivial)
|
2014-01-05 19:03:35 +00:00
|
|
|
print Environment 1
|
2013-12-22 22:10:42 +00:00
|
|
|
Variable b : Bool
|
|
|
|
Definition a := b
|
2014-01-05 18:32:47 +00:00
|
|
|
Theorem T : b => a := (by (* imp_tac() .. normalize_tac() .. assumption_tac() *))
|