Skip to content

Commit 107bef7

Browse files
committed
fix: add not actually redundant simp
1 parent 7a8fd25 commit 107bef7

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Init/Data/Fin/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -918,7 +918,7 @@ theorem exists_fin_succ {P : Fin (n + 1) → Prop} : (∃ i, P i) ↔ P 0 ∨
918918
@[simp] theorem forall_fin_zero {p : Fin 0Prop} : (∀ i, p i) ↔ True :=
919919
fun _ => trivial, fun _ ⟨_, h⟩ => False.elim <| Nat.not_lt_zero _ h⟩
920920

921-
theorem exists_fin_zero {p : Fin 0Prop} : (∃ i, p i) ↔ False := by simp
921+
@[simp] theorem exists_fin_zero {p : Fin 0Prop} : (∃ i, p i) ↔ False := by simp
922922

923923
@[simp] theorem forall_fin_one {p : Fin 1Prop} : (∀ i, p i) ↔ p 0 :=
924924
fun h => h _, fun h i => Subsingleton.elim i 0 ▸ h⟩

0 commit comments

Comments
 (0)