Skip to content

Commit c3fe021

Browse files
committed
specialize the fixpoint combinator
1 parent 840c675 commit c3fe021

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Init/Internal/ExtrinsicTermination.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -31,7 +31,7 @@ variable {α : Sort _} {β : α → Sort _} {C : α → Sort _} {C₂ : (a : α)
3131

3232
namespace Std.Internal
3333

34-
@[always_inline]
34+
@[specialize]
3535
public partial def opaqueFix [∀ x, Nonempty (C x)] (F : (x : α) → ((y : α) → C y) → C x) (x : α) : C x :=
3636
F x (opaqueFix F)
3737

@@ -61,7 +61,7 @@ public def extrinsicFix_eq [∀ x, Nonempty (C x)] {F : (x : α) → ((y : α)
6161
rw [WellFounded.fix_eq, show (extrinsicFix F) = (fun y => extrinsicFix F y) by rfl]
6262
simp only [extrinsicFix, dif_pos h, h.choose_spec.choose_spec.2]
6363

64-
@[always_inline]
64+
@[specialize]
6565
public partial def opaqueFix₂ [∀ a b, Nonempty (C₂ a b)]
6666
(F : (a : α) → (b : β a) → ((a' : α) → (b' : β a') → C₂ a' b') → C₂ a b) (a : α) (b : β a) :
6767
C₂ a b :=

0 commit comments

Comments
 (0)