We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent b038fd1 commit 3e3ab44Copy full SHA for 3e3ab44
Batteries/Data/Fin/Lemmas.lean
@@ -11,16 +11,6 @@ namespace Fin
11
12
attribute [norm_cast] val_last
13
14
--- Forward port from lean4#10627
15
-@[simp] theorem forall_fin_zero {P : Fin 0 → Prop} : (∀ i, P i) ↔ True := by
16
- rw [iff_true]; intro ⟨_, _⟩; contradiction
17
-
18
19
-@[simp] theorem exists_fin_zero {P : Fin 0 → Prop} : (∃ i, P i) ↔ False := by simp
20
21
22
-attribute [simp] exists_fin_one forall_fin_one exists_fin_two forall_fin_two
23
24
/-! ### foldl/foldr -/
25
26
theorem foldl_assoc {op : α → α → α} [ha : Std.Associative op] {f : Fin n → α} {a₁ a₂} :
0 commit comments