Skip to content

Commit

Permalink
Merge PR coq#17920: ssrbool: reenable overwriting-delimiting-key
Browse files Browse the repository at this point in the history
Reviewed-by: proux01
Co-authored-by: proux01 <[email protected]>
  • Loading branch information
coqbot-app[bot] and proux01 authored Dec 4, 2023
2 parents ababbf4 + 5fe1563 commit 691049e
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions theories/ssr/ssrbool.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,8 +15,6 @@
Require Bool.
Require Import ssreflect ssrfun.

#[export] Set Warnings "-overwriting-delimiting-key".

(**
A theory of boolean predicates and operators. A large part of this file is
concerned with boolean reflection.
Expand Down Expand Up @@ -468,7 +466,9 @@ Reserved Notation "[ ==> b1 , b2 , .. , bn => c ]" (at level 0, format
"'[hv' [ ==> '[' b1 , '/' b2 , '/' .. , '/' bn ']' '/' => c ] ']'").

(** Shorter delimiter **)
#[export] Set Warnings "-overwriting-delimiting-key".
Delimit Scope bool_scope with B.
#[export] Set Warnings "overwriting-delimiting-key".
Open Scope bool_scope.

(** An alternative to xorb that behaves somewhat better wrt simplification. **)
Expand Down

0 comments on commit 691049e

Please sign in to comment.