summaryrefslogtreecommitdiff
path: root/test-suite/success/rewrite_in.v
blob: 29fe915ff49548af77139d7040362cd9870e9254 (plain)
1
2
3
4
5
6
7
8
Require Import Setoid.

Goal forall (P Q : Prop) (f:P->Prop) (p:P), (P<->Q) -> f p -> True.
  intros P Q f p H.
  rewrite H in p || trivial.
Qed.