Skip to content

Commit

Permalink
Adapt to Coq PR #18845 fixing an issue with maximal implicit argument…
Browse files Browse the repository at this point in the history
…s for notations.

The new (originally intended) behaviour for selecting maximal implicit
arguments of a notation for an applied constant in the presence of
multiple signatures of implicit arguments. Such notations now behave
like ordinary constants or abbreviations for non applied constants,
that is, they complete the application with as much implicit arguments
as possible.

This impacts the notation "naturality[ x ] := (@Naturality _ _ _ _ x)"
which is now resolved with 3 trailing implicit arguments, making
tactics such as a "srewrite (naturality[foo])" failing with unresolved
arguments.

It happens that the "naturality" constant mostly uses one signature of
implicit arguments. So, the adaptation is to restrict "naturality" to
only this signature.
  • Loading branch information
herbelin committed Dec 30, 2023
1 parent 4427c02 commit 5089fc0
Showing 1 changed file with 4 additions and 6 deletions.
10 changes: 4 additions & 6 deletions Theory/Natural/Transformation.v
Original file line number Diff line number Diff line change
Expand Up @@ -46,10 +46,8 @@ Qed.
End Transform.

Arguments transform {_ _ _ _} _ _.
Arguments naturality
{_ _ _ _ _ _ _ _}, {_ _ _ _} _ {_ _ _}, {_ _ _ _} _ _ _ _.
Arguments naturality_sym
{_ _ _ _ _ _ _ _}, {_ _ _ _} _ {_ _ _}, {_ _ _ _} _ _ _ _.
Arguments naturality {_ _ _ _} _ _ _ _.
Arguments naturality_sym {_ _ _ _} _ _ _ _.

Declare Scope transform_scope.
Declare Scope transform_type_scope.
Expand Down Expand Up @@ -214,8 +212,8 @@ Program Definition whisker_right {C D : Category} {F G : C ⟶ D} `(N : F ⟹ G)
{E : Category} (X : E ⟶ C) : F ◯ X ⟹ G ◯ X := {|
transform := λ x, N (X x);

naturality := λ _ _ _, naturality;
naturality_sym := λ _ _ _, naturality_sym
naturality := λ _ _ _, naturality _ _ _ _;
naturality_sym := λ _ _ _, naturality_sym _ _ _ _
|}.

Notation "N ⊲ F" := (whisker_right N F) (at level 10).
Expand Down

0 comments on commit 5089fc0

Please sign in to comment.