We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent f33a3a8 commit c57f62bCopy full SHA for c57f62b
src/Data/Rational/Base.agda
@@ -222,7 +222,7 @@ p@record{} * q@record{} = (↥ p ℤ.* ↥ q) / (↧ₙ p ℕ.* ↧ₙ q)
222
223
-- subtraction
224
_-_ : ℚ → ℚ → ℚ
225
-p@record{} - q@record{} = p + (- q)
+p - q = p + (- q)
226
227
-- reciprocal: requires a proof that the numerator is not zero
228
1/_ : (p : ℚ) → .{{_ : NonZero p}} → ℚ
@@ -231,7 +231,7 @@ p@record{} - q@record{} = p + (- q)
231
232
-- division: requires a proof that the denominator is not zero
233
_÷_ : (p q : ℚ) → .{{_ : NonZero q}} → ℚ
234
-p@record{} ÷ q@record{} = p * (1/ q)
+p ÷ q = p * (1/ q)
235
236
-- max
237
_⊔_ : (p q : ℚ) → ℚ
0 commit comments