Skip to content

Commit 3e3ab44

Browse files
committed
1 parent b038fd1 commit 3e3ab44

File tree

1 file changed

+0
-10
lines changed

1 file changed

+0
-10
lines changed

Batteries/Data/Fin/Lemmas.lean

Lines changed: 0 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -11,16 +11,6 @@ namespace Fin
1111

1212
attribute [norm_cast] val_last
1313

14-
-- Forward port from lean4#10627
15-
@[simp] theorem forall_fin_zero {P : Fin 0Prop} : (∀ i, P i) ↔ True := by
16-
rw [iff_true]; intro ⟨_, _⟩; contradiction
17-
18-
-- Forward port from lean4#10627
19-
@[simp] theorem exists_fin_zero {P : Fin 0Prop} : (∃ i, P i) ↔ False := by simp
20-
21-
-- Forward port from lean4#10627
22-
attribute [simp] exists_fin_one forall_fin_one exists_fin_two forall_fin_two
23-
2414
/-! ### foldl/foldr -/
2515

2616
theorem foldl_assoc {op : α → α → α} [ha : Std.Associative op] {f : Fin n → α} {a₁ a₂} :

0 commit comments

Comments
 (0)