File tree Expand file tree Collapse file tree 2 files changed +2
-3
lines changed Expand file tree Collapse file tree 2 files changed +2
-3
lines changed Original file line number Diff line number Diff line change @@ -1415,7 +1415,6 @@ private
1415
1415
| [1+m]⊖[1+n]≡m⊖n (m ℕ.+ o ℕ.* suc m) (m ℕ.+ n ℕ.* suc m)
1416
1416
| +-cancelˡ-⊖ m (o ℕ.* suc m) (n ℕ.* suc m)
1417
1417
| ⊖-≥ n≤o
1418
- | +-comm (- (+ (m ℕ.+ n ℕ.* suc m))) (+ (m ℕ.+ o ℕ.* suc m))
1419
1418
| ⊖-≥ (ℕ.*-mono-≤ n≤o (ℕ.≤-refl {x = suc m}))
1420
1419
| ℕ.*-distribʳ-∸ (suc m) o n
1421
1420
| +◃n≡+n (o ℕ.* suc m ∸ n ℕ.* suc m)
Original file line number Diff line number Diff line change @@ -111,8 +111,8 @@ module _ (descent : Descent _<_ P) where
111
111
h<P (suc n) = g<P n
112
112
113
113
Π[P∘h] : ∀ n → P (h n)
114
- Π[P∘h] zero rewrite g0≡z = py
115
- Π[P∘h] (suc n) = Π[P∘g] n
114
+ Π[P∘h] zero = py
115
+ Π[P∘h] (suc n) = Π[P∘g] n
116
116
117
117
descent∧wf⇒infiniteDescent : WellFounded _<_ → InfiniteDescent _<_ P
118
118
descent∧wf⇒infiniteDescent wf = descent∧acc⇒infiniteDescentFrom (wf _)
You can’t perform that action at this time.
0 commit comments