aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3735.v
blob: 00886cbc605bf23e3a01796561bb77df5186b271 (plain)
1
2
3
4
Require Import Coq.Program.Tactics.
Class Foo := { bar : Type }.
Fail Lemma foo : Foo -> bar. (* 'Command has indeed failed.' in both 8.4 and trunk *)
Fail Program Lemma foo : Foo -> bar.