Skip to content

Commit

Permalink
Merge pull request #137 from herbelin/master+adapt-coq-pr18445-fix-ap…
Browse files Browse the repository at this point in the history
…plied-notations-multiple-implicit
  • Loading branch information
jwiegley authored Jan 9, 2024
2 parents 41ab38d + 5089fc0 commit e50af05
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 e50af05

Please sign in to comment.