diff options
Diffstat (limited to 'test-suite/success/destruct.v')
-rw-r--r-- | test-suite/success/destruct.v | 4 |
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/success/destruct.v b/test-suite/success/destruct.v index f5848ffe0..2aa07cde1 100644 --- a/test-suite/success/destruct.v +++ b/test-suite/success/destruct.v @@ -393,6 +393,10 @@ intros * Heq H Heq'. destruct H. Abort. +Goal 2=1 -> 1=0. +intro H. destruct H. +Fail (match goal with n:nat |- _ => unfold n end). (* Check that no let-in remains *) + (* Check clearing of names *) Inductive eqnat (x : nat) : nat -> Prop := |