DEBSOURCES
Skip Quicknav
sources / coq / 8.20.1%2Bdfsg-1 / test-suite / bugs / bug_3212.v
12345678910
Lemma H : Prop = Prop. reflexivity. Qed. Lemma foo : match H in (_ = X) return X with | eq_refl => True end. Proof. Fail destruct H. Abort.