aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/6313.v
blob: 1715e7f90657382d5ca2e98af55a1e7d5979a084 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
(* Former open goals in nested proofs were lost *)

Inductive foo := a | b | c.
Goal foo -> foo.
  intro x.
  simple refine (match x with
                 | a => _
                 | b => ltac:(exact b)
                 | c => _
                 end); [exact a|exact c].
Abort.

(* Another example *)

Goal (True/\0=0 -> True) -> True.
  intro f.
  refine
   (f ltac:(split; only 1:exact I)).
  reflexivity.
Qed.