summaryrefslogtreecommitdiff
path: root/test-suite/success/shrink_abstract.v
blob: 916bb846a9b3f2635b2e0d64d3d296bf1bf41d7a (plain)
1
2
3
4
5
6
7
8
9
10
11
Definition foo : forall (n m : nat), bool.
Proof.
pose (p := 0).
intros n.
pose (q := n).
intros m.
pose (r := m).
abstract (destruct m; [left|right]).
Defined.

Check (foo_subproof : nat -> bool).