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.
≤-Reasoning
1 parent 032506d commit 850cb99Copy full SHA for 850cb99
src/Data/Nat/Divisibility.agda
@@ -42,7 +42,6 @@ open import Data.Nat.Divisibility.Core public hiding (*-pres-∣)
42
module _ (m∣n : m ∣ n) where
43
44
open _∣_ m∣n
45
- open ≤-Reasoning
46
47
quotient≢0 : .{{NonZero n}} → NonZero quotient
48
quotient≢0 rewrite equality = m*n≢0⇒m≢0 quotient
@@ -59,13 +58,16 @@ module _ (m∣n : m ∣ n) where
59
58
m <⟨ m<n ⟩
60
n ≡⟨ equalityᵒ ⟩
61
m * quotient ∎
+ where open ≤-Reasoning
62
63
quotient-< : .{{NonTrivial m}} → .{{NonZero n}} → quotient < n
64
quotient-< = begin-strict
65
quotient <⟨ m<m*n quotient m (nonTrivial⇒n>1 m) ⟩
66
quotient * m ≡⟨ equality ⟨
67
n ∎
68
- where instance _ = quotient≢0
+ where
69
+ open ≤-Reasoning
70
+ instance _ = quotient≢0
71
72
-- Exports
73
0 commit comments