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/N07_Prod.lean

42 lines
1.0 KiB
Plaintext

2 years ago
import TestGame.Metadata
import Mathlib.Algebra.Module.Submodule.Lattice
import Mathlib.Data.Real.Basic
import Mathlib.LinearAlgebra.Span
Game "TestGame"
World "Module2"
Level 7
Title "Lineare Abbildung"
Introduction
"
Die externe Summe von (Unter-) Modulen wird als `V × W` geschrieben
Das Produkt zweier Module wird mit `×` geschrieben.
Lean weiss dann automatisch, dass das Produkt wieder ein Vektorraum ist.
-/
example : module ( × ) := infer_instance
/-
Und ` × ` und `fin 2 → ` sind natürlich Isomorph. In Praxis eignet sich
die Funktionsschreibweise besser, deshalb verwenden wir diese als
definition für `ℝ²`.
Hier die Äquivalenz als generelle Typen:
-/
example : (fin 2 → ) ≃ × :=
begin
apply pi_fin_two_equiv,
end
/-
Äquivalenz als Vektorräume schreibt man als ``-lineare Äquivalenz `≃ₗ[]`.
"
Statement
"Zeige dass das Produkt ` × ` und `ℝ²` isomorph sind als ``-Vektorräume."
: ((Fin 2) → ) ≃ₗ[] × := by
sorry