@@ -31,7 +31,27 @@ Bug-fixes
31
31
32
32
* The following operators were missing a fixity declaration, which has now
33
33
been fixed -
34
- ```
34
+ ```
35
+ infix -1 _$ⁿ_ (Data.Vec.N-ary)
36
+ infix 4 _≋_ (Data.Vec.Functional.Relation.Binary.Equality.Setoid)
37
+ infix 4 _≟_ (Reflection.AST.Definition)
38
+ infix 4 _≡ᵇ_ (Reflection.AST.Literal)
39
+ infix 4 _≈?_ _≟_ _≈_ (Reflection.AST.Meta)
40
+ infix 4 _≈?_ _≟_ _≈_ (Reflection.AST.Name)
41
+ infix 4 _≟-Telescope_ (Reflection.AST.Term)
42
+ infix 4 _≟_ (Reflection.AST.Argument.Information)
43
+ infix 4 _≟_ (Reflection.AST.Argument.Modality)
44
+ infix 4 _≟_ (Reflection.AST.Argument.Quantity)
45
+ infix 4 _≟_ (Reflection.AST.Argument.Relevance)
46
+ infix 4 _≟_ (Reflection.AST.Argument.Visibility)
47
+ infixr 8 _^_ (Function.Endomorphism.Propositional)
48
+ infixr 8 _^_ (Function.Endomorphism.Setoid)
49
+ infix 4 _≃_ (Function.HalfAdjointEquivalence)
50
+ infix 4 _≈_ _≈ᵢ_ _≤_ (Function.Metric.Bundles)
51
+ infixl 6 _∙_ (Function.Metric.Bundles)
52
+ infix 4 _≈_ (Function.Metric.Nat.Bundles)
53
+ infix 3 _←_ _↢_ (Function.Related)
54
+
35
55
infix 4 _ℕ<_ _ℕ≤infinity _ℕ≤_ (Codata.Sized.Conat)
36
56
infix 6 _ℕ+_ _+ℕ_ (Codata.Sized.Conat)
37
57
infixl 4 _+ _* (Data.List.Kleene.Base)
0 commit comments