Skip to content

Commit 850cb99

Browse files
committed
localised use of ≤-Reasoning
1 parent 032506d commit 850cb99

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

src/Data/Nat/Divisibility.agda

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -42,7 +42,6 @@ open import Data.Nat.Divisibility.Core public hiding (*-pres-∣)
4242
module _ (m∣n : m ∣ n) where
4343

4444
open _∣_ m∣n
45-
open ≤-Reasoning
4645

4746
quotient≢0 : .{{NonZero n}} NonZero quotient
4847
quotient≢0 rewrite equality = m*n≢0⇒m≢0 quotient
@@ -59,13 +58,16 @@ module _ (m∣n : m ∣ n) where
5958
m <⟨ m<n ⟩
6059
n ≡⟨ equalityᵒ ⟩
6160
m * quotient ∎
61+
where open ≤-Reasoning
6262

6363
quotient-< : .{{NonTrivial m}} .{{NonZero n}} quotient < n
6464
quotient-< = begin-strict
6565
quotient <⟨ m<m*n quotient m (nonTrivial⇒n>1 m) ⟩
6666
quotient * m ≡⟨ equality ⟨
6767
n ∎
68-
where instance _ = quotient≢0
68+
where
69+
open ≤-Reasoning
70+
instance _ = quotient≢0
6971

7072
-- Exports
7173

0 commit comments

Comments
 (0)