File: bug_19138.v

package info (click to toggle)
coq 8.20.1%2Bdfsg-1
  • links: PTS, VCS
  • area: main
  • in suites: forky, sid, trixie
  • size: 44,116 kB
  • sloc: ml: 234,160; sh: 4,301; python: 3,270; ansic: 2,644; makefile: 882; lisp: 172; javascript: 63; xml: 24; sed: 2
file content (21 lines) | stat: -rw-r--r-- 554 bytes parent folder | download | duplicates (2)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
From Ltac2 Require Import Ltac2 Constr.
Import Constr.Unsafe.

Goal True.
  let t := open_constr:(_ :> False) in
  match kind t with
  | Evar e _ => Control.new_goal e > [refine 'I|]
  | _ => Control.throw Not_found
  end.
  Show Existentials. (* Existential 1 = ?Goal : [ |- False] (shelved) *)
Abort.

Goal True.
  let t := unshelve open_constr:(_ :> False) in
  Control.extend [Control.shelve] (fun () => ()) [];
  match kind t with
  | Evar e _ => Control.new_goal e > [refine 'I|]
  | _ => Control.throw Not_found
  end.
  Show Existentials.
Abort.