summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/6910.v
blob: 5167a5364a97d13913c4c6ccab96d75b06080b50 (plain)
1
2
3
4
5
From Coq Require Import ssreflect ssrfun.

(* We should be able to use Some_inj as a view: *)
Lemma foo (x y : nat) : Some x = Some y -> x = y.
Proof. by move/Some_inj. Qed.