Skip to content

Commit cb7d162

Browse files
committed
feat: (v +ᵥ s) -ᵥ (v +ᵥ t) = s -ᵥ t (#21058)
From PFR
1 parent ace1a06 commit cb7d162

File tree

1 file changed

+9
-2
lines changed

1 file changed

+9
-2
lines changed

Mathlib/Algebra/AddTorsor.lean

Lines changed: 9 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -38,6 +38,8 @@ multiplicative group actions).
3838
3939
-/
4040

41+
open scoped Pointwise
42+
4143
/-- An `AddTorsor G P` gives a structure to the nonempty type `P`,
4244
acted on by an `AddGroup G` with a transitive and free action given
4345
by the `+ᵥ` operation and a corresponding subtraction given by the
@@ -162,8 +164,6 @@ theorem vadd_eq_vadd_iff_neg_add_eq_vsub {v₁ v₂ : G} {p₁ p₂ : P} :
162164

163165
namespace Set
164166

165-
open Pointwise
166-
167167
theorem singleton_vsub_self (p : P) : ({p} : Set P) -ᵥ {p} = {(0 : G)} := by
168168
rw [Set.singleton_vsub_singleton, vsub_self]
169169

@@ -231,6 +231,13 @@ theorem vadd_eq_vadd_iff_sub_eq_vsub {v₁ v₂ : G} {p₁ p₂ : P} :
231231
theorem vsub_sub_vsub_comm (p₁ p₂ p₃ p₄ : P) : p₁ -ᵥ p₂ - (p₃ -ᵥ p₄) = p₁ -ᵥ p₃ - (p₂ -ᵥ p₄) := by
232232
rw [← vsub_vadd_eq_vsub_sub, vsub_vadd_comm, vsub_vadd_eq_vsub_sub]
233233

234+
namespace Set
235+
236+
@[simp] lemma vadd_set_vsub_vadd_set (v : G) (s t : Set P) : (v +ᵥ s) -ᵥ (v +ᵥ t) = s -ᵥ t := by
237+
ext; simp [mem_vsub, mem_vadd_set]
238+
239+
end Set
240+
234241
end comm
235242

236243
namespace Prod

0 commit comments

Comments
 (0)