summaryrefslogtreecommitdiff
path: root/test-suite/success/extraction_polyprop.v
blob: 936d838c50e657bb931fe68040438d1343bbf44f (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
(* The current extraction cannot handle this situation,
   and shouldn't try, otherwise it might produce some Ocaml
   code that segfaults. See Table.error_singleton_become_prop
   or S. Glondu's thesis for more details. *)

Require Coq.extraction.Extraction.

Definition f {X} (p : (nat -> X) * True) : X * nat :=
  (fst p 0, 0).

Definition f_prop := f ((fun _ => I),I).

Fail Extraction f_prop.