aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_4412.v
blob: a1fb3de4dba078b323db26c9b5e4aaee2dcbb7d0 (plain)
1
2
3
4
5
Require Import Coq.Bool.Bool Coq.Setoids.Setoid.
Goal forall (P : forall b : bool, b = true -> Type) (x y : bool) (H : andb x y = true) (H' : P _ H), True.
  intros.
  Fail rewrite Bool.andb_true_iff in H.
Abort.