File tree Expand file tree Collapse file tree 1 file changed +9
-2
lines changed Expand file tree Collapse file tree 1 file changed +9
-2
lines changed Original file line number Diff line number Diff line change @@ -38,6 +38,8 @@ multiplicative group actions).
38
38
39
39
-/
40
40
41
+ open scoped Pointwise
42
+
41
43
/-- An `AddTorsor G P` gives a structure to the nonempty type `P`,
42
44
acted on by an `AddGroup G` with a transitive and free action given
43
45
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} :
162
164
163
165
namespace Set
164
166
165
- open Pointwise
166
-
167
167
theorem singleton_vsub_self (p : P) : ({p} : Set P) -ᵥ {p} = {(0 : G)} := by
168
168
rw [Set.singleton_vsub_singleton, vsub_self]
169
169
@@ -231,6 +231,13 @@ theorem vadd_eq_vadd_iff_sub_eq_vsub {v₁ v₂ : G} {p₁ p₂ : P} :
231
231
theorem vsub_sub_vsub_comm (p₁ p₂ p₃ p₄ : P) : p₁ -ᵥ p₂ - (p₃ -ᵥ p₄) = p₁ -ᵥ p₃ - (p₂ -ᵥ p₄) := by
232
232
rw [← vsub_vadd_eq_vsub_sub, vsub_vadd_comm, vsub_vadd_eq_vsub_sub]
233
233
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
+
234
241
end comm
235
242
236
243
namespace Prod
You can’t perform that action at this time.
0 commit comments