Skip to content

Commit 4b42cd1

Browse files
Fix level for FixPoint in Induction.WellFounded (#1265)
1 parent b6c7856 commit 4b42cd1

File tree

2 files changed

+4
-1
lines changed

2 files changed

+4
-1
lines changed

CHANGELOG.md

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -18,6 +18,9 @@ Bug-fixes
1818
* Fixed various algebraic bundles not correctly re-exporting
1919
`commutativeSemigroup` proofs.
2020

21+
* Fix in `Induction.WellFounded.FixPoint`, where the well-founded relation `_<_` and
22+
the predicate `P` were required to live at the same universe level.
23+
2124
Non-backwards compatible changes
2225
--------------------------------
2326

src/Induction/WellFounded.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -106,7 +106,7 @@ module All {_<_ : Rel A r} (wf : WellFounded _<_) ℓ where
106106
#-}
107107

108108
module FixPoint
109-
{_<_ : Rel A } (wf : WellFounded _<_)
109+
{_<_ : Rel A r} (wf : WellFounded _<_)
110110
(P : Pred A ℓ) (f : WfRec _<_ P ⊆′ P)
111111
(f-ext : (x : A) {IH IH′ : WfRec _<_ P x} ( {y} y<x IH y y<x ≡ IH′ y y<x) f x IH ≡ f x IH′)
112112
where

0 commit comments

Comments
 (0)