File tree Expand file tree Collapse file tree 2 files changed +4
-4
lines changed
List/Relation/Binary/Sublist/Propositional/Example Expand file tree Collapse file tree 2 files changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -14,8 +14,8 @@ open import Relation.Binary.PropositionalEquality using (_≡_; refl; sym; cong;
14
14
open ≡-Reasoning
15
15
16
16
open import Data.List using (List; []; _∷_; [_])
17
- open import Data.List.All using (Null; [])
18
17
open import Data.List.Membership.Propositional using (_∈_)
18
+ open import Data.List.Relation.Unary.All using (Null; [])
19
19
open import Data.List.Relation.Binary.Sublist.Propositional using
20
20
( _⊆_; []; _∷_; _∷ʳ_
21
21
; ⊆-refl; ⊆-trans; minimum
Original file line number Diff line number Diff line change @@ -778,14 +778,14 @@ private
778
778
+-monoʳ-< : ∀ x → (x +_) Preserves _<_ ⟶ _<_
779
779
+-monoʳ-< x y<z = +-mono-≤-< (≤-refl {x}) y<z
780
780
781
- x≤y+x : ∀ ( x y) → x ≤ y + x
781
+ x≤y+x : ∀ x y → x ≤ y + x
782
782
x≤y+x x y = begin
783
783
x ≡⟨ sym (+-identityˡ x) ⟩
784
784
0ᵇ + x ≤⟨ +-monoˡ-≤ x (0≤x y) ⟩
785
785
y + x ∎
786
786
where open ≤-Reasoning
787
787
788
- x≤x+y : ∀ ( x y) → x ≤ x + y
788
+ x≤x+y : ∀ x y → x ≤ x + y
789
789
x≤x+y x y = begin
790
790
x ≤⟨ x≤y+x x y ⟩
791
791
y + x ≡⟨ +-comm y x ⟩
@@ -1318,7 +1318,7 @@ suc-* x y = begin
1318
1318
x + x * y ∎
1319
1319
where open ≡-Reasoning
1320
1320
1321
- x≤suc[y]*x : ∀ ( x y) → x ≤ (suc y) * x
1321
+ x≤suc[y]*x : ∀ x y → x ≤ (suc y) * x
1322
1322
x≤suc[y]*x x y = begin
1323
1323
x ≤⟨ x≤x+y x (y * x) ⟩
1324
1324
x + y * x ≡⟨ sym (suc-* y x) ⟩
You can’t perform that action at this time.
0 commit comments