Skip to content

Commit 78a871c

Browse files
Saransh-cppandreasabel
authored andcommitted
Add more fixities (#2008)
1 parent c7f6db7 commit 78a871c

File tree

9 files changed

+35
-0
lines changed

9 files changed

+35
-0
lines changed

CHANGELOG.md

+8
Original file line numberDiff line numberDiff line change
@@ -112,6 +112,14 @@ Bug-fixes
112112
infix 4 _≈∙_ (Relation.Binary.Construct.Add.Point.Equality)
113113
infix 4 _≤⁺_ _≤⊤⁺ (Relation.Binary.Construct.Add.Supremum.NonStrict)
114114
infixr 5 _∷ʳ_ (Relation.Binary.Construct.Closure.Transitive)
115+
infixr 5 _∷_ (Codata.Guarded.Stream.Relation.Unary.All)
116+
infixr 5 _∷_ (Foreign.Haskell.List.NonEmpty)
117+
infix 4 _≈_ (Function.Metric.Rational.Bundles)
118+
infixl 6 _ℕ+_ (Level.Literals)
119+
infixr 6 _∪_ (Relation.Binary.Construct.Union)
120+
infixl 6 _+ℤ_ (Relation.Binary.HeterogeneousEquality.Quotients.Examples)
121+
infix 4 _≉_ _≈ᵢ_ _≤ᵢ_ (Relation.Binary.Indexed.Homogeneous.Bundles)
122+
infixr 5 _∷ᴹ_ _∷⁻¹ᴹ_ (Text.Regex.Search)
115123
```
116124

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

src/Codata/Guarded/Stream/Relation/Unary/All.agda

+2
Original file line numberDiff line numberDiff line change
@@ -20,6 +20,8 @@ private
2020
P Q R : Pred A p
2121
xs : Stream A
2222

23+
infixr 5 _∷_
24+
2325
record All (P : Pred A ℓ) (as : Stream A) : Setwhere
2426
coinductive
2527
constructor _∷_

src/Foreign/Haskell/List/NonEmpty.agda

+2
Original file line numberDiff line numberDiff line change
@@ -25,5 +25,7 @@ private
2525
data NonEmpty (A : Set a) : Set a where
2626
_∷_ : A List A NonEmpty A
2727

28+
infixr 5 _∷_
29+
2830
{-# FOREIGN GHC type AgdaNonEmpty l a = NE.NonEmpty a #-}
2931
{-# COMPILE GHC NonEmpty = data AgdaNonEmpty ((NE.:|)) #-}

src/Function/Metric/Rational/Bundles.agda

+12
Original file line numberDiff line numberDiff line change
@@ -34,6 +34,8 @@ record ProtoMetric a ℓ : Set (suc (a ⊔ ℓ)) where
3434
d : DistanceFunction Carrier
3535
isProtoMetric : IsProtoMetric _≈_ d
3636

37+
infix 4 _≈_
38+
3739
open IsProtoMetric isProtoMetric public
3840

3941
------------------------------------------------------------------------
@@ -46,6 +48,8 @@ record PreMetric a ℓ : Set (suc (a ⊔ ℓ)) where
4648
d : DistanceFunction Carrier
4749
isPreMetric : IsPreMetric _≈_ d
4850

51+
infix 4 _≈_
52+
4953
open IsPreMetric isPreMetric public
5054

5155
protoMetric : ProtoMetric a ℓ
@@ -63,6 +67,8 @@ record QuasiSemiMetric a ℓ : Set (suc (a ⊔ ℓ)) where
6367
d : DistanceFunction Carrier
6468
isQuasiSemiMetric : IsQuasiSemiMetric _≈_ d
6569

70+
infix 4 _≈_
71+
6672
open IsQuasiSemiMetric isQuasiSemiMetric public
6773

6874
preMetric : PreMetric a ℓ
@@ -83,6 +89,8 @@ record SemiMetric a ℓ : Set (suc (a ⊔ ℓ)) where
8389
d : DistanceFunction Carrier
8490
isSemiMetric : IsSemiMetric _≈_ d
8591

92+
infix 4 _≈_
93+
8694
open IsSemiMetric isSemiMetric public
8795

8896
quasiSemiMetric : QuasiSemiMetric a ℓ
@@ -103,6 +111,8 @@ record Metric a ℓ : Set (suc (a ⊔ ℓ)) where
103111
d : DistanceFunction Carrier
104112
isMetric : IsMetric _≈_ d
105113

114+
infix 4 _≈_
115+
106116
open IsMetric isMetric public
107117

108118
semiMetric : SemiMetric a ℓ
@@ -123,6 +133,8 @@ record UltraMetric a ℓ : Set (suc (a ⊔ ℓ)) where
123133
d : DistanceFunction Carrier
124134
isUltraMetric : IsUltraMetric _≈_ d
125135

136+
infix 4 _≈_
137+
126138
open IsUltraMetric isUltraMetric public
127139

128140
semiMetric : SemiMetric a ℓ

src/Level/Literals.agda

+2
Original file line numberDiff line numberDiff line change
@@ -15,6 +15,8 @@ open import Level using (Level; 0ℓ)
1515

1616
-- Increase a Level by a number of sucs.
1717

18+
infixl 6 _ℕ+_
19+
1820
_ℕ+_ : Level Level
1921
zero ℕ+ ℓ =
2022
suc n ℕ+ ℓ = Level.suc (n ℕ+ ℓ)

src/Relation/Binary/Construct/Union.agda

+2
Original file line numberDiff line numberDiff line change
@@ -24,6 +24,8 @@ private
2424
------------------------------------------------------------------------
2525
-- Definition
2626

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

src/Relation/Binary/HeterogeneousEquality/Quotients/Examples.agda

+2
Original file line numberDiff line numberDiff line change
@@ -82,6 +82,8 @@ module Integers (quot : Quotients 0ℓ 0ℓ) where
8282
module _ (ext : {a b} {A : Set a} {B₁ B₂ : A Set b} {f₁ : a B₁ a}
8383
{f₂ : a B₂ a} ( a f₁ a ≅ f₂ a) f₁ ≅ f₂) where
8484

85+
infixl 6 _+ℤ_
86+
8587
_+ℤ_ :
8688
_+ℤ_ = Properties₂.lift₂ ext Int Int (λ i j abs (i +² j))
8789
$ λ {a} {b} {c} p p′ compat-abs (+²-cong {a} {b} {c} p p′)

src/Relation/Binary/Indexed/Homogeneous/Bundles.agda

+3
Original file line numberDiff line numberDiff line change
@@ -39,6 +39,8 @@ record IndexedSetoid {i} (I : Set i) c ℓ : Set (suc (i ⊔ c ⊔ ℓ)) where
3939
Carrier : Set _
4040
Carrier = i Carrierᵢ i
4141

42+
infix 4 _≉_
43+
4244
_≈_ : B.Rel Carrier _
4345
_≈_ = Lift Carrierᵢ _≈ᵢ_
4446

@@ -103,6 +105,7 @@ record IndexedPreorder {i} (I : Set i) c ℓ₁ ℓ₂ :
103105

104106
record IndexedPoset {i} (I : Set i) c ℓ₁ ℓ₂ :
105107
Set (suc (i ⊔ c ⊔ ℓ₁ ⊔ ℓ₂)) where
108+
infix 4 _≈ᵢ_ _≤ᵢ_
106109
field
107110
Carrierᵢ : I Set c
108111
_≈ᵢ_ : IRel Carrierᵢ ℓ₁

src/Text/Regex/Search.agda

+2
Original file line numberDiff line numberDiff line change
@@ -87,6 +87,8 @@ module Prefix where
8787
[]⁻¹ᴹ : {e} Match (Prefix _≡_) [] e [] ∈ e
8888
[]⁻¹ᴹ (mkMatch .[] p []) = p
8989

90+
infixr 5 _∷ᴹ_ _∷⁻¹ᴹ_
91+
9092
_∷ᴹ_ : {xs e} x Match (Prefix _≡_) xs (eat x e) Match (Prefix _≡_) (x ∷ xs) e
9193
x ∷ᴹ (mkMatch ys ys∈e\x ys≤xs) = mkMatch (x ∷ ys) (eat-sound x _ ys∈e\x) (refl ∷ ys≤xs)
9294

0 commit comments

Comments
 (0)