Skip to content

Commit

Permalink
Fixed deprecation warnings in Data.Bin.Properties
Browse files Browse the repository at this point in the history
  • Loading branch information
MatthewDaggitt committed Sep 22, 2019
1 parent da0d91b commit a9b3af3
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Data/Bin/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -77,7 +77,7 @@ as 1# ≟ bs 1# with as ≟ₑ bs
1+ (m₁ +ℕ n₁ *ℕ 2) ≤⟨ s≤s (ℕₚ.+-monoˡ-≤ _ (𝔽ₚ.toℕ≤pred[n] a)) ⟩
1+ (1 +ℕ n₁ *ℕ 2) ≡⟨ refl ⟩
1+ n₁ *ℕ 2 ≤⟨ ℕₚ.*-mono-≤ lt ℕₚ.≤-refl ⟩
n₂ *ℕ 2 ≤⟨ ℕₚ.n≤m+n m₂ (n₂ *ℕ 2) ⟩
n₂ *ℕ 2 ≤⟨ ℕₚ.m≤n+m (n₂ *ℕ 2) m₂
m₂ +ℕ n₂ *ℕ 2 ∎)
where
open ℕₚ.≤-Reasoning
Expand All @@ -94,7 +94,7 @@ as 1# ≟ bs 1# with as ≟ₑ bs
m₁ = Fin.toℕ a; m₂ = Fin.toℕ b; n = toℕ (bs 1#)

1<[23] : {b} [] 1# < (b ∷ []) 1#
1<[23] {b} = less (ℕₚ.n≤m+n (Fin.toℕ b) 2)
1<[23] {b} = less (ℕₚ.m≤n+m 2 (Fin.toℕ b))

1<2+ : {b bs} [] 1# < (b ∷ bs) 1#
1<2+ {_} {[]} = 1<[23]
Expand Down

0 comments on commit a9b3af3

Please sign in to comment.