File: decidable.v

package info (click to toggle)
coq-stdpp 1.11.0-1
  • links: PTS, VCS
  • area: main
  • in suites: forky, sid, trixie
  • size: 1,696 kB
  • sloc: makefile: 52; sh: 35; sed: 1
file content (11 lines) | stat: -rw-r--r-- 408 bytes parent folder | download
1
2
3
4
5
6
7
8
9
10
11
From stdpp Require Import list.

(** Test that Coq does not infer [x ∈ xs] as [False] by eagerly using
[False_dec] on a goal with unresolved type class instances. *)
Example issue_165 (x : nat) :
  ¬ ∃ xs : list nat, (guard (x ∈ xs);; Some x) ≠ None.
Proof.
  intros [xs Hxs]. case_guard; [|done].
  Fail done. (* Would succeed if the instance backing [x ∈ xs] is inferred as
  [False]. *)
Abort.