5b25da8c43
closes #358
28 lines
549 B
Text
28 lines
549 B
Text
open nat
|
|
|
|
example (x y : nat) (H : (fun (a : nat), sigma.pr1 ⟨a, y⟩) x = 0) : x = 0 :=
|
|
begin
|
|
esimp at H,
|
|
exact H
|
|
end
|
|
|
|
definition foo [irreducible] (a : nat) := a
|
|
|
|
example (x y : nat) (H : (fun (a : nat), sigma.pr1 ⟨foo a, y⟩) x = 0) : x = 0 :=
|
|
begin
|
|
esimp ↑foo at H,
|
|
exact H
|
|
end
|
|
|
|
example (x y : nat) (H : x = 0) : (fun (a : nat), sigma.pr1 ⟨foo a, y⟩) x = 0 :=
|
|
begin
|
|
esimp ↑foo,
|
|
exact H
|
|
end
|
|
|
|
example (x y : nat) (H : x = 0) : (fun (a : nat), sigma.pr1 ⟨foo a, y⟩) x = 0 :=
|
|
begin
|
|
esimp,
|
|
unfold foo,
|
|
exact H
|
|
end
|