File tree Expand file tree Collapse file tree 2 files changed +4
-1
lines changed Expand file tree Collapse file tree 2 files changed +4
-1
lines changed Original file line number Diff line number Diff line change @@ -18,6 +18,9 @@ Bug-fixes
18
18
* Fixed various algebraic bundles not correctly re-exporting
19
19
` commutativeSemigroup ` proofs.
20
20
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
+
21
24
Non-backwards compatible changes
22
25
--------------------------------
23
26
Original file line number Diff line number Diff line change @@ -106,7 +106,7 @@ module All {_<_ : Rel A r} (wf : WellFounded _<_) ℓ where
106
106
#-}
107
107
108
108
module FixPoint
109
- {_<_ : Rel A ℓ } (wf : WellFounded _<_)
109
+ {_<_ : Rel A r } (wf : WellFounded _<_)
110
110
(P : Pred A ℓ) (f : WfRec _<_ P ⊆′ P)
111
111
(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′)
112
112
where
You can’t perform that action at this time.
0 commit comments