Skip to content

Commit 2cdbd56

Browse files
committed
fix: knock-ons from agda#2168
1 parent cceb530 commit 2cdbd56

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

src/Data/Rational/Unnormalised/Properties.agda

+4-4
Original file line numberDiff line numberDiff line change
@@ -746,7 +746,7 @@ neg⇒nonZero (mkℚᵘ (-[1+ _ ]) _) = _
746746
+-identityˡ p = ≃-reflexive (+-identityˡ-≡ p)
747747

748748
+-identityʳ-≡ : RightIdentity _≡_ 0ℚᵘ _+_
749-
+-identityʳ-≡ = comm+idˡ⇒idʳ +-comm-≡ {e = 0ℚᵘ} +-identityˡ-≡
749+
+-identityʳ-≡ = commidˡ⇒idʳ +-comm-≡ {e = 0ℚᵘ} +-identityˡ-≡
750750

751751
+-identityʳ : RightIdentity _≃_ 0ℚᵘ _+_
752752
+-identityʳ p = ≃-reflexive (+-identityʳ-≡ p)
@@ -1104,7 +1104,7 @@ p≤q⇒0≤q-p {p} {q} p≤q = begin
11041104
*-identityˡ-≡ p@record{} = ↥↧≡⇒≡ (ℤ.*-identityˡ (↥ p)) (ℕ.+-identityʳ (↧ₙ p))
11051105

11061106
*-identityʳ-≡ : RightIdentity _≡_ 1ℚᵘ _*_
1107-
*-identityʳ-≡ = comm+idˡ⇒idʳ *-comm-≡ {e = 1ℚᵘ} *-identityˡ-≡
1107+
*-identityʳ-≡ = commidˡ⇒idʳ *-comm-≡ {e = 1ℚᵘ} *-identityˡ-≡
11081108

11091109
*-identity-≡ : Identity _≡_ 1ℚᵘ _*_
11101110
*-identity-≡ = *-identityˡ-≡ , *-identityʳ-≡
@@ -1144,7 +1144,7 @@ p≤q⇒0≤q-p {p} {q} p≤q = begin
11441144
*-zeroˡ p@record{} = *≡* refl
11451145

11461146
*-zeroʳ : RightZero _≃_ 0ℚᵘ _*_
1147-
*-zeroʳ = Consequences.comm+zeˡ⇒zeʳ ≃-setoid *-comm *-zeroˡ
1147+
*-zeroʳ = Consequences.commzeˡ⇒zeʳ ≃-setoid *-comm *-zeroˡ
11481148

11491149
*-zero : Zero _≃_ 0ℚᵘ _*_
11501150
*-zero = *-zeroˡ , *-zeroʳ
@@ -1171,7 +1171,7 @@ invertible⇒≄ {p} {q} (1/p-q , 1/x*x≃1 , x*1/x≃1) p≃q = 0≄1 (begin
11711171
in *≡* eq where open ℤ-solver
11721172

11731173
*-distribʳ-+ : _DistributesOverʳ_ _≃_ _*_ _+_
1174-
*-distribʳ-+ = Consequences.comm+distrˡ⇒distrʳ ≃-setoid +-cong *-comm *-distribˡ-+
1174+
*-distribʳ-+ = Consequences.commdistrˡ⇒distrʳ ≃-setoid +-cong *-comm *-distribˡ-+
11751175

11761176
*-distrib-+ : _DistributesOver_ _≃_ _*_ _+_
11771177
*-distrib-+ = *-distribˡ-+ , *-distribʳ-+

0 commit comments

Comments
 (0)