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
14151415 | [1+m]⊖[1+n]≡m⊖n (m ℕ.+ o ℕ.* suc m) (m ℕ.+ n ℕ.* suc m)
14161416 | +-cancelˡ-⊖ m (o ℕ.* suc m) (n ℕ.* suc m)
14171417 | ⊖-≥ n≤o
1418- | +-comm (- (+ (m ℕ.+ n ℕ.* suc m))) (+ (m ℕ.+ o ℕ.* suc m))
14191418 | ⊖-≥ (ℕ.*-mono-≤ n≤o (ℕ.≤-refl {x = suc m}))
14201419 | ℕ.*-distribʳ-∸ (suc m) o n
14211420 | +◃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
111111 h<P (suc n) = g<P n
112112
113113 Π[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
116116
117117 descent∧wf⇒infiniteDescent : WellFounded _<_ → InfiniteDescent _<_ P
118118 descent∧wf⇒infiniteDescent wf = descent∧acc⇒infiniteDescentFrom (wf _)
You can’t perform that action at this time.
0 commit comments