Skip to content

Commit b10b384

Browse files
committed
postpone @[inline] annotations to later PR
1 parent 01aa996 commit b10b384

File tree

2 files changed

+0
-3
lines changed

2 files changed

+0
-3
lines changed

src/Init/Prelude.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1098,7 +1098,6 @@ until `c` is known.
10981098
| Or.inl h => hp h
10991099
| Or.inr h => hq h
11001100

1101-
@[inline]
11021101
instance [dp : Decidable p] : Decidable (Not p) :=
11031102
match dp with
11041103
| isTrue hp => isFalse (absurd hp)

src/Init/PropLemmas.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -448,14 +448,12 @@ theorem Decidable.by_contra [Decidable p] : (¬p → False) → p := of_not_not
448448
@[expose] protected def Or.by_cases' [Decidable q] {α : Sort u} (h : p ∨ q) (h₁ : p → α) (h₂ : q → α) : α :=
449449
if hq : q then h₂ hq else h₁ (h.resolve_right hq)
450450

451-
@[inline]
452451
instance exists_prop_decidable {p} (P : p → Prop)
453452
[Decidable p] [∀ h, Decidable (P h)] : Decidable (∃ h, P h) :=
454453
if h : p then
455454
decidable_of_decidable_of_iff ⟨fun h2 => ⟨h, h2⟩, fun ⟨_, h2⟩ => h2⟩
456455
else isFalse fun ⟨h', _⟩ => h h'
457456

458-
@[inline]
459457
instance forall_prop_decidable {p} (P : p → Prop)
460458
[Decidable p] [∀ h, Decidable (P h)] : Decidable (∀ h, P h) :=
461459
if h : p then

0 commit comments

Comments
 (0)