summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/6631.v
blob: 100dc13fc8d7b0320a114f35889a6f0014a226c4 (plain)
1
2
3
4
5
6
7
Require Import Coq.derive.Derive.

Derive f SuchThat (f = 1 + 1) As feq.
Proof.
  transitivity 2; [refine (eq_refl 2)|].
  transitivity 2.
  2:abstract exact (eq_refl 2).