You cannot select more than 25 topics Topics must start with a letter or number, can include dashes ('-') and can be up to 35 characters long.
lean4game/server/testgame/TestGame/Levels/LinearAlgebra/N06_Sum.lean

26 lines
544 B
Plaintext

2 years ago
import TestGame.Metadata
import Mathlib.Algebra.Module.Submodule.Lattice
import Mathlib.LinearAlgebra.Span
open Submodule
Game "TestGame"
World "Module2"
Level 6
Title "Lineare Abbildung"
Introduction
"
Eine interne Summe über eine Familie von Untermodulen `(T : ι → submodule K V)`
wird als `⨆ (i : ι), T i` geschrieben (`\\supr`).
"
Statement
""
{K V ι : Type _} [Field K] [AddCommMonoid V] [Module K V]
(T : ι → Submodule K V) : (⨆ (i : ι), T i) = span K ( i, T i) := by
rw [Submodule.span_unionᵢ]
simp