aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2019-04-05 15:11:54 -0400
committerGravatar Jason Gross <jgross@mit.edu>2019-04-05 15:11:54 -0400
commitccbbf7e5593e0d3a646528c6629668c64a1d86e4 (patch)
treea28dc3a25e69e1f35d46a35f09af5e2efc244083
parent2172994d31ffc63bb27bc558d2861285fba45e40 (diff)
Hint reflect on negb
This way we can pick it up based on the bool, and not just on the Prop. This allows us to `apply Reflect.reflect_bool in H` for `H : negb (_ =? _) = true` and have it work.
-rw-r--r--src/Util/Bool/Reflect.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/src/Util/Bool/Reflect.v b/src/Util/Bool/Reflect.v
index 8a5333f0a..0d31853fe 100644
--- a/src/Util/Bool/Reflect.v
+++ b/src/Util/Bool/Reflect.v
@@ -161,6 +161,7 @@ Proof. exact _. Qed.
(** Disallow infinite loops of reflect_not *)
Hint Extern 0 (reflect (~?A) _) => eapply (@reflect_not A) : typeclass_instances.
+Hint Extern 0 (reflect _ (negb ?b)) => eapply (@reflect_not _ b) : typeclass_instances.
Global Instance reflect_eq_unit : reflect_rel (@eq unit) (fun _ _ => true) | 10. exact _. Qed.
Global Instance reflect_eq_bool : reflect_rel (@eq bool) Bool.eqb | 10. exact _. Qed.