File tree Expand file tree Collapse file tree 8 files changed +20
-0
lines changed Expand file tree Collapse file tree 8 files changed +20
-0
lines changed Original file line number Diff line number Diff line change @@ -105,6 +105,13 @@ Bug-fixes
105
105
infix 8 _⁻¹ (Data.Parity.Base)
106
106
infixr 5 _`∷_ (Data.Vec.Reflection)
107
107
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)
108
115
```
109
116
110
117
* In ` System.Exit ` , the ` ExitFailure ` constructor is now carrying an integer
Original file line number Diff line number Diff line change @@ -176,6 +176,8 @@ mutual
176
176
177
177
-- Equality is weakly decidable.
178
178
179
+ infix 4 _≟H_ _≟N_
180
+
179
181
_≟H_ : ∀ {n} → WeaklyDecidable (_≈H_ {n = n})
180
182
∅ ≟H ∅ = just ∅
181
183
∅ ≟H (_ *x+ _) = nothing
Original file line number Diff line number Diff line change @@ -21,6 +21,7 @@ open import Relation.Binary.Structures
21
21
------------------------------------------------------------------------
22
22
23
23
record PartialSetoid a ℓ : Set (suc (a ⊔ ℓ)) where
24
+ infix 4 _≈_
24
25
field
25
26
Carrier : Set a
26
27
_≈_ : Rel Carrier ℓ
Original file line number Diff line number Diff line change @@ -28,6 +28,8 @@ import Relation.Nullary.Decidable as Dec
28
28
------------------------------------------------------------------------
29
29
-- Definition
30
30
31
+ infix 4 _<₋_
32
+
31
33
data _<₋_ : Rel (A ₋) (a ⊔ ℓ) where
32
34
⊥₋<[_] : (l : A) → ⊥₋ <₋ [ l ]
33
35
[_] : {k l : A} → k < l → [ k ] <₋ [ l ]
Original file line number Diff line number Diff line change @@ -24,6 +24,8 @@ import Relation.Nullary.Decidable as Dec
24
24
------------------------------------------------------------------------
25
25
-- Definition
26
26
27
+ infix 4 _≈∙_
28
+
27
29
data _≈∙_ : Rel (Pointed A) (a ⊔ ℓ) where
28
30
∙≈∙ : ∙ ≈∙ ∙
29
31
[_] : {k l : A} → k ≈ l → [ k ] ≈∙ [ l ]
Original file line number Diff line number Diff line change @@ -26,6 +26,8 @@ import Relation.Binary.Construct.Add.Supremum.Equality as Equality
26
26
------------------------------------------------------------------------
27
27
-- Definition
28
28
29
+ infix 4 _≤⁺_ _≤⊤⁺
30
+
29
31
data _≤⁺_ : Rel (A ⁺) (a ⊔ ℓ) where
30
32
[_] : {k l : A} → k ≤ l → [ k ] ≤⁺ [ l ]
31
33
_≤⊤⁺ : (k : A ⁺) → k ≤⁺ ⊤⁺
Original file line number Diff line number Diff line change @@ -39,6 +39,8 @@ module _ {_∼_ : Rel A ℓ} where
39
39
private
40
40
_∼⁺_ = TransClosure _∼_
41
41
42
+ infixr 5 _∷ʳ_
43
+
42
44
_∷ʳ_ : ∀ {x y z} → (x∼⁺y : x ∼⁺ y) (y∼z : y ∼ z) → x ∼⁺ z
43
45
[ x∼y ] ∷ʳ y∼z = x∼y ∷ [ y∼z ]
44
46
(x∼y ∷ x∼⁺y) ∷ʳ y∼z = x∼y ∷ (x∼⁺y ∷ʳ y∼z)
Original file line number Diff line number Diff line change @@ -24,6 +24,8 @@ private
24
24
------------------------------------------------------------------------
25
25
-- Definition
26
26
27
+ infixl 6 _∩_
28
+
27
29
_∩_ : REL A B ℓ₁ → REL A B ℓ₂ → REL A B (ℓ₁ ⊔ ℓ₂)
28
30
L ∩ R = λ i j → L i j × R i j
29
31
You can’t perform that action at this time.
0 commit comments