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/adam/Adam/Levels/LinearAlgebra/M04_Basis.lean

33 lines
518 B
Plaintext

import Adam.Metadata
2 years ago
import Mathlib.Algebra.Module.Submodule.Lattice
2 years ago
import Mathlib
2 years ago
Game "Adam"
2 years ago
World "Basis"
Level 4
Title "Basis"
2 years ago
namespace Ex_Basis
scoped notation "ℝ²" => Fin 2 →
open Submodule
2 years ago
Introduction
"
"
2 years ago
lemma exercise1 : LinearIndependent ![(![1, 0] : ℝ²), ![1, 1]] := sorry
lemma exercise2 : ≤ span (Set.range ![(![1, 0] : Fin 2 → ), ![1, 1]]) := sorry
Statement : Basis (Fin 2) ℝ² := by
apply Basis.mk
apply exercise1
apply exercise2
end Ex_Basis