summaryrefslogtreecommitdiff
path: root/test-suite/vio/seff.v
blob: 447e7798336a56989a7b9f44037378215ba48a00 (plain)
1
2
3
4
5
6
7
8
9
10
Inductive equal T (x : T) : T -> Type := Equal : equal T x x.

Module bla.

Lemma test n : equal nat n (n + n) -> equal nat (n + n + n) n.
Proof using.
intro H. rewrite <- H. rewrite <- H. exact (Equal nat n).
Qed.

End bla.