Skip to content

Commit

Permalink
Move reservation of notations .1 and .2 from ssr to Init
Browse files Browse the repository at this point in the history
Also move them from level 2 to level 1 in preparation
of removal of camlp5 recovery mechanism.
  • Loading branch information
proux01 committed Oct 30, 2023
1 parent bda17b6 commit 7861b99
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 2 deletions.
5 changes: 5 additions & 0 deletions theories/Init/Notations.v
Original file line number Diff line number Diff line change
Expand Up @@ -114,6 +114,11 @@ Notation "'if' c 'is' p 'then' u 'else' v" :=

End IfNotations.

(** Notations for first and second projections *)

Reserved Notation "p .1" (at level 1, left associativity, format "p .1").
Reserved Notation "p .2" (at level 1, left associativity, format "p .2").

(** Scopes *)

Declare Scope core_scope.
Expand Down
2 changes: 0 additions & 2 deletions theories/ssr/ssrfun.v
Original file line number Diff line number Diff line change
Expand Up @@ -225,8 +225,6 @@ Unset Strict Implicit.
Unset Printing Implicit Defensive.

(** Parsing / printing declarations. *)
Reserved Notation "p .1" (at level 2, left associativity, format "p .1").
Reserved Notation "p .2" (at level 2, left associativity, format "p .2").
Reserved Notation "f ^~ y" (at level 10, y at level 8, no associativity,
format "f ^~ y").
Reserved Notation "@^~ x" (at level 10, x at level 8, no associativity,
Expand Down

0 comments on commit 7861b99

Please sign in to comment.