summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3920.v
blob: a4adb23cc2c6c7ca022be82b6f8b8a62011a704a (plain)
1
2
3
4
5
6
7
Require Import Setoid.
Axiom P : nat -> Prop.
Axiom P_or : forall x y, P (x + y) <-> P x \/ P y.
Lemma foo (H : P 3) : False.
eapply or_introl in H.
erewrite <- P_or in H.
(* Error: No such hypothesis: H *)