lean2/tests/lean/cast1.lean
Leonardo de Moura c0c2f52087 Add Cast, DomInj and RanInj. Improve operator << for lean_frontend objects.
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-09-06 18:32:15 -07:00

20 lines
709 B
Text

Variable vector : Type -> Nat -> Type
Axiom N0 (n : Nat) : n + 0 = n
Theorem V0 (T : Type) (n : Nat) : (vector T (n + 0)) = (vector T n) :=
Congr (Refl (vector T)) (N0 n)
Variable f (n : Nat) (v : vector Int n) : Int
Variable m : Nat
Variable v1 : vector Int (m + 0)
(*
The following application will fail because (vector Int (m + 0)) and (vector Int m)
are not definitionally equal.
*)
Check f m v1
(*
The next one succeeds using the "casting" operator.
We can do it, because (V0 Int m) is a proof that
(vector Int (m + 0)) and (vector Int m) are propositionally equal.
That is, they have the same interpretation in the lean set theoretic
semantics.
*)
Check f m (cast (V0 Int m) v1)