@@ -232,7 +232,7 @@ lemma single_apply_left {f : α → β} (hf : function.injective f)
232
232
single (f x) y (f z) = single x y z :=
233
233
by { classical, simp only [single_apply, hf.eq_iff] }
234
234
235
- lemma single_eq_indicator : ⇑(single a b) = set.indicator {a} (λ _, b) :=
235
+ lemma single_eq_set_indicator : ⇑(single a b) = set.indicator {a} (λ _, b) :=
236
236
by { classical, ext, simp [single_apply, set.indicator, @eq_comm _ a] }
237
237
238
238
@[simp] lemma single_eq_same : (single a b : α →₀ M) a = b :=
@@ -242,7 +242,7 @@ by { classical, exact pi.single_eq_same a b }
242
242
by { classical, exact pi.single_eq_of_ne' h _ }
243
243
244
244
lemma single_eq_update [decidable_eq α] (a : α) (b : M) : ⇑(single a b) = function.update 0 a b :=
245
- by rw [single_eq_indicator , ← set.piecewise_eq_indicator, set.piecewise_singleton]
245
+ by rw [single_eq_set_indicator , ← set.piecewise_eq_indicator, set.piecewise_singleton]
246
246
247
247
lemma single_eq_pi_single [decidable_eq α] (a : α) (b : M) : ⇑(single a b) = pi.single a b :=
248
248
single_eq_update a b
@@ -284,7 +284,7 @@ have (single a b₁ : α →₀ M) a = (single a b₂ : α →₀ M) a, by rw eq
284
284
by rwa [single_eq_same, single_eq_same] at this
285
285
286
286
lemma single_apply_eq_zero {a x : α} {b : M} : single a b x = 0 ↔ (x = a → b = 0 ) :=
287
- by simp [single_eq_indicator ]
287
+ by simp [single_eq_set_indicator ]
288
288
289
289
lemma single_apply_ne_zero {a x : α} {b : M} : single a b x ≠ 0 ↔ (x = a ∧ b ≠ 0 ) :=
290
290
by simp [single_apply_eq_zero]
@@ -337,7 +337,7 @@ lemma support_single_disjoint {b' : M} (hb : b ≠ 0) (hb' : b' ≠ 0) {i j : α
337
337
by rw [support_single_ne_zero _ hb, support_single_ne_zero _ hb', disjoint_singleton]
338
338
339
339
@[simp] lemma single_eq_zero : single a b = 0 ↔ b = 0 :=
340
- by simp [ext_iff, single_eq_indicator ]
340
+ by simp [ext_iff, single_eq_set_indicator ]
341
341
342
342
lemma single_swap (a₁ a₂ : α) (b : M) : single a₁ b a₂ = single a₂ b a₁ :=
343
343
by { classical, simp only [single_apply], ac_refl }
0 commit comments