Skip to content

Commit a0b06ba

Browse files
authored
Add infix declartions to exists syntax (#1340)
1 parent f0ef8a6 commit a0b06ba

File tree

2 files changed

+6
-0
lines changed

2 files changed

+6
-0
lines changed

CHANGELOG.md

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -164,3 +164,5 @@ Other minor additions
164164
```agda
165165
+-*-commutativeSemiring : CommutativeSemiring 0ℓ 0ℓ
166166
```
167+
168+
* Added infix declarations to `Data.Product.∃-syntax` and `Data.Product.∄-syntax`.

src/Data/Product.agda

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -75,11 +75,15 @@ _,′_ = _,_
7575

7676
-- Syntax
7777

78+
infix 2 ∃-syntax
79+
7880
∃-syntax : {A : Set a} (A Set b) Set (a ⊔ b)
7981
∃-syntax =
8082

8183
syntax ∃-syntax (λ x B) = ∃[ x ] B
8284

85+
infix 2 ∄-syntax
86+
8387
∄-syntax : {A : Set a} (A Set b) Set (a ⊔ b)
8488
∄-syntax =
8589

0 commit comments

Comments
 (0)