Commit a23e4d4
committed
feat(LinearAlgebra/AffineSpace/AffineSubspace/Basic):
Add two lemmas about affine maps applied to the infimum of two subspaces, similar to lemmas that exist for various other subobject types.
```lean
lemma map_inf_le (s₁ s₂ : AffineSubspace k P₁) : (s₁ ⊓ s₂).map f ≤ s₁.map f ⊓ s₂.map f :=
```
```lean
lemma map_inf_eq (hf : Function.Injective f) (s₁ s₂ : AffineSubspace k P₁) :
(s₁ ⊓ s₂).map f = s₁.map f ⊓ s₂.map f := by
```map_inf lemmas (#32015)1 parent 9e28bbc commit a23e4d4
1 file changed
+9
-0
lines changedLines changed: 9 additions & 0 deletions
| Original file line number | Diff line number | Diff line change | |
|---|---|---|---|
| |||
561 | 561 | | |
562 | 562 | | |
563 | 563 | | |
| 564 | + | |
| 565 | + | |
| 566 | + | |
| 567 | + | |
| 568 | + | |
| 569 | + | |
| 570 | + | |
| 571 | + | |
| 572 | + | |
564 | 573 | | |
565 | 574 | | |
566 | 575 | | |
| |||
0 commit comments