summaryrefslogtreecommitdiff
path: root/test-suite/bugs/opened/3311.v
blob: 1c66bc1e55dc3e3b06fc9110d0327e8fe014b7d5 (plain)
1
2
3
4
5
6
7
8
9
10
Require Import Setoid.
Axiom bar : True = False.
Goal True.
  Fail setoid_rewrite bar. (* Toplevel input, characters 15-33:
Error:
Tactic failure:setoid rewrite failed: Unable to satisfy the rewriting constraints.

Could not find an instance for "subrelation eq (Basics.flip Basics.impl)".
With the following constraints:
?3 : "True" *)