aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Rename.v
blob: 8a5db157c0330022fe55be3b2122726062c12371 (plain)
1
2
3
4
5
Goal forall n : nat, n = 0 -> n = 0.
intros.
rename n into p.
induction p; auto.
Qed.