Skip to content

Commit c5771cf

Browse files
Fixed Data.Nat.Binary.Properties propertis
1 parent ae02ebb commit c5771cf

File tree

2 files changed

+4
-4
lines changed

2 files changed

+4
-4
lines changed

src/Data/List/Relation/Binary/Sublist/Propositional/Example/UniqueBoundVariables.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -14,8 +14,8 @@ open import Relation.Binary.PropositionalEquality using (_≡_; refl; sym; cong;
1414
open ≡-Reasoning
1515

1616
open import Data.List using (List; []; _∷_; [_])
17-
open import Data.List.All using (Null; [])
1817
open import Data.List.Membership.Propositional using (_∈_)
18+
open import Data.List.Relation.Unary.All using (Null; [])
1919
open import Data.List.Relation.Binary.Sublist.Propositional using
2020
( _⊆_; []; _∷_; _∷ʳ_
2121
; ⊆-refl; ⊆-trans; minimum

src/Data/Nat/Binary/Properties.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -778,14 +778,14 @@ private
778778
+-monoʳ-< : x (x +_) Preserves _<_ ⟶ _<_
779779
+-monoʳ-< x y<z = +-mono-≤-< (≤-refl {x}) y<z
780780

781-
x≤y+x : (x y) x ≤ y + x
781+
x≤y+x : x y x ≤ y + x
782782
x≤y+x x y = begin
783783
x ≡⟨ sym (+-identityˡ x) ⟩
784784
0ᵇ + x ≤⟨ +-monoˡ-≤ x (0≤x y) ⟩
785785
y + x ∎
786786
where open ≤-Reasoning
787787

788-
x≤x+y : (x y) x ≤ x + y
788+
x≤x+y : x y x ≤ x + y
789789
x≤x+y x y = begin
790790
x ≤⟨ x≤y+x x y ⟩
791791
y + x ≡⟨ +-comm y x ⟩
@@ -1318,7 +1318,7 @@ suc-* x y = begin
13181318
x + x * y ∎
13191319
where open ≡-Reasoning
13201320

1321-
x≤suc[y]*x : (x y) x ≤ (suc y) * x
1321+
x≤suc[y]*x : x y x ≤ (suc y) * x
13221322
x≤suc[y]*x x y = begin
13231323
x ≤⟨ x≤x+y x (y * x) ⟩
13241324
x + y * x ≡⟨ sym (suc-* y x) ⟩

0 commit comments

Comments
 (0)