summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1100.v
blob: 6d619c74863d36b9e3ae03121db3e1685716d9ef (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.