Skip to content

Commit a671ae3

Browse files
authored
Fixities for Relation and Algebra (#1992)
1 parent ad8c039 commit a671ae3

File tree

8 files changed

+20
-0
lines changed

8 files changed

+20
-0
lines changed

CHANGELOG.md

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -105,6 +105,13 @@ Bug-fixes
105105
infix 8 _⁻¹ (Data.Parity.Base)
106106
infixr 5 _`∷_ (Data.Vec.Reflection)
107107
infixr 5 _∷=_ (Data.Vec.Membership.Setoid)
108+
infix 4 _≟H_ _≟N_ (Algebra.Solver.Ring)
109+
infix 4 _≈_ (Relation.Binary.Bundles)
110+
infixl 6 _∩_ (Relation.Binary.Construct.Intersection)
111+
infix 4 _<₋_ (Relation.Binary.Construct.Add.Infimum.Strict)
112+
infix 4 _≈∙_ (Relation.Binary.Construct.Add.Point.Equality)
113+
infix 4 _≤⁺_ _≤⊤⁺ (Relation.Binary.Construct.Add.Supremum.NonStrict)
114+
infixr 5 _∷ʳ_ (Relation.Binary.Construct.Closure.Transitive)
108115
```
109116

110117
* In `System.Exit`, the `ExitFailure` constructor is now carrying an integer

src/Algebra/Solver/Ring.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -176,6 +176,8 @@ mutual
176176

177177
-- Equality is weakly decidable.
178178

179+
infix 4 _≟H_ _≟N_
180+
179181
_≟H_ : {n} WeaklyDecidable (_≈H_ {n = n})
180182
∅ ≟H ∅ = just ∅
181183
∅ ≟H (_ *x+ _) = nothing

src/Relation/Binary/Bundles.agda

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -21,6 +21,7 @@ open import Relation.Binary.Structures
2121
------------------------------------------------------------------------
2222

2323
record PartialSetoid a ℓ : Set (suc (a ⊔ ℓ)) where
24+
infix 4 _≈_
2425
field
2526
Carrier : Set a
2627
_≈_ : Rel Carrier ℓ

src/Relation/Binary/Construct/Add/Infimum/Strict.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -28,6 +28,8 @@ import Relation.Nullary.Decidable as Dec
2828
------------------------------------------------------------------------
2929
-- Definition
3030

31+
infix 4 _<₋_
32+
3133
data _<₋_ : Rel (A ₋) (a ⊔ ℓ) where
3234
⊥₋<[_] : (l : A) ⊥₋ <₋ [ l ]
3335
[_] : {k l : A} k < l [ k ] <₋ [ l ]

src/Relation/Binary/Construct/Add/Point/Equality.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -24,6 +24,8 @@ import Relation.Nullary.Decidable as Dec
2424
------------------------------------------------------------------------
2525
-- Definition
2626

27+
infix 4 _≈∙_
28+
2729
data _≈∙_ : Rel (Pointed A) (a ⊔ ℓ) where
2830
∙≈∙ : ∙ ≈∙ ∙
2931
[_] : {k l : A} k ≈ l [ k ] ≈∙ [ l ]

src/Relation/Binary/Construct/Add/Supremum/NonStrict.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -26,6 +26,8 @@ import Relation.Binary.Construct.Add.Supremum.Equality as Equality
2626
------------------------------------------------------------------------
2727
-- Definition
2828

29+
infix 4 _≤⁺_ _≤⊤⁺
30+
2931
data _≤⁺_ : Rel (A ⁺) (a ⊔ ℓ) where
3032
[_] : {k l : A} k ≤ l [ k ] ≤⁺ [ l ]
3133
_≤⊤⁺ : (k : A ⁺) k ≤⁺ ⊤⁺

src/Relation/Binary/Construct/Closure/Transitive.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -39,6 +39,8 @@ module _ {_∼_ : Rel A ℓ} where
3939
private
4040
_∼⁺_ = TransClosure _∼_
4141

42+
infixr 5 _∷ʳ_
43+
4244
_∷ʳ_ : {x y z} (x∼⁺y : x ∼⁺ y) (y∼z : y ∼ z) x ∼⁺ z
4345
[ x∼y ] ∷ʳ y∼z = x∼y ∷ [ y∼z ]
4446
(x∼y ∷ x∼⁺y) ∷ʳ y∼z = x∼y ∷ (x∼⁺y ∷ʳ y∼z)

src/Relation/Binary/Construct/Intersection.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -24,6 +24,8 @@ private
2424
------------------------------------------------------------------------
2525
-- Definition
2626

27+
infixl 6 _∩_
28+
2729
_∩_ : REL A B ℓ₁ REL A B ℓ₂ REL A B (ℓ₁ ⊔ ℓ₂)
2830
L ∩ R = λ i j L i j × R i j
2931

0 commit comments

Comments
 (0)