diff options
| author | Gaëtan Gilbert | 2018-12-13 22:13:52 +0100 |
|---|---|---|
| committer | Gaëtan Gilbert | 2018-12-13 22:13:52 +0100 |
| commit | 7e3603069cf591c6c70ef25d4cfc72f62aa44058 (patch) | |
| tree | e2559c13bba99ffe058bb9c54c27e2974f59f018 | |
| parent | 4e88b488230959ef82a3b1cd0bbf601078b33d04 (diff) | |
| parent | 9304f93c18485965af1507be71cf0a86d1758d4b (diff) | |
Merge PR #9193: Tests for #4509, #6202 which happen to be fixed (was a lost of evars in shelf)
| -rw-r--r-- | test-suite/bugs/closed/bug_4509.v | 11 | ||||
| -rw-r--r-- | test-suite/bugs/closed/bug_6202.v | 11 |
2 files changed, 22 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/bug_4509.v b/test-suite/bugs/closed/bug_4509.v new file mode 100644 index 0000000000..ceae7c5fc3 --- /dev/null +++ b/test-suite/bugs/closed/bug_4509.v @@ -0,0 +1,11 @@ +(* Was solved at some time, suspectingly in PR #6328 *) + +Goal exists n, n > 1. +Proof. + unshelve eexists. (*2 goals, as expected*) + Undo. + unshelve (eexists; instantiate (1:=ltac:(idtac))). (*only 1 goal*) + shelve. + Undo. + 2:unshelve instantiate (1:=_). +Abort. diff --git a/test-suite/bugs/closed/bug_6202.v b/test-suite/bugs/closed/bug_6202.v new file mode 100644 index 0000000000..899260f59a --- /dev/null +++ b/test-suite/bugs/closed/bug_6202.v @@ -0,0 +1,11 @@ +(* This was fixed at some time, suspectingly in PR #6328 *) + +Inductive foo := F (a : forall var : Type -> Type, unit -> var unit) (_ : a = a). +Goal foo. + eexists (fun var => fun u : unit => ltac:(clear u)). + shelve. + Unshelve. + all:[ > | ]. + shelve. + Fail Grab Existential Variables. +Abort. |
