summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/1100.v
blob: 32c78b4b9e9a27ba134fba8ee6ce7b50d1a6bf69 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
Require Import Setoid.

Parameter P : nat -> Prop.
Parameter Q : nat -> Prop.
Parameter PQ : forall n, P n <-> Q n.

Lemma PQ2 : forall n, P n -> Q n.
  intros.
  rewrite PQ in H.
  trivial.
Qed.