lean2/tests/lean/sig6.lean

8 lines
514 B
Text
Raw Normal View History

variables A B : (Type U)
variables t1 t2 : A B
axiom pair_Ax {A : (Type U)} {B : A → (Type U)} (p : sig x, B x) : (tuple (sig x, B x) : (proj1 p), (proj2 p)) = p
theorem spairext {A B : (Type U)} {p1 p2 : A B} (H1 : proj1 p1 = proj1 p2) (H2 : proj2 p1 = proj2 p2) : p1 = p2
:= calc p1 = tuple (proj1 p1), (proj2 p1) : symm (pair_Ax p1)
... = tuple (proj1 p2), (proj2 p1) : { H1 }
... = tuple (proj1 p2), (proj2 p2) : { H2 }
... = p2 : pair_Ax p2