44a31dd8fb
- The extension does not have to be provided. - It can also import Lua files. - Hierachical names can be used instead of strings. Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
12 lines
431 B
Text
12 lines
431 B
Text
Import tactic
|
|
SetOption pp::implicit true
|
|
SetOption pp::coercion true
|
|
SetOption pp::notation false
|
|
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
|
|
Definition D := read V1 1 (by trivial)
|
|
Show Environment 1
|
|
Variable b : Bool
|
|
Definition a := b
|
|
Theorem T : b => a := (by (** imp_tac() .. normalize_tac() .. assumption_tac() **))
|