Skip to content

Commit

Permalink
properties curryFin + interior product definition (know its a bit mes…
Browse files Browse the repository at this point in the history
…sy to do this in this branch but well...)
  • Loading branch information
MetalCreator666 committed Jan 24, 2025
1 parent d80bdbe commit b92dabc
Show file tree
Hide file tree
Showing 2 changed files with 19 additions and 0 deletions.
15 changes: 15 additions & 0 deletions DeRhamCohomology/ContinuousAlternatingMap/Curry.lean
Original file line number Diff line number Diff line change
Expand Up @@ -102,6 +102,21 @@ def curryFin (f : E [⋀^Fin (n + 1)]→L[𝕜] F) : E →L[𝕜] E [⋀^Fin n]
apply le_of_eq
exact ContinuousMultilinearMap.curryLeft_norm f.toContinuousMultilinearMap

theorem curryFin_apply (f : E [⋀^Fin (n + 1)]→L[𝕜] F) (x : E) (m : Fin n → E) :
curryFin f x m = f (Fin.cons x m) :=
rfl

theorem curryFin_add (f g : E [⋀^Fin (n + 1)]→L[𝕜] F) :
curryFin (f + g) = curryFin f + curryFin g := by
ext e v
simp [curryFin_apply]

theorem curryFin_smul {M : Type*} [Monoid M] [DistribMulAction M F] [ContinuousConstSMul M F]
[SMulCommClass 𝕜 M F] (c : M) (f : E [⋀^Fin (n + 1)]→L[𝕜] F) :
curryFin (c • f) = c • curryFin f := by
ext e v
simp [curryFin_apply]

variable [DecidableEq ι] [DecidableEq ι']

/-- summand used in `ContinuousAlternatingMap.uncurrySum` -/
Expand Down
4 changes: 4 additions & 0 deletions DeRhamCohomology/DifferentialForm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -210,6 +210,10 @@ theorem pullback_constOfIsEmpty (f : E → F) (g : G) :
pullback f (constOfIsEmpty g) = fun _ ↦ (ContinuousAlternatingMap.constOfIsEmpty ℝ E (Fin 0) g) :=
rfl

/- Interior product of differential forms -/
def iprod (ω : Ω^(m + 1)⟮E, F⟯) (v : E → E) : Ω^m⟮E, F⟯ :=
fun e => ContinuousAlternatingMap.curryFin (ω e) (v e)

/- Wedge product of differential forms -/
def wedge_product (ω₁ : Ω^m⟮E, F⟯) (ω₂ : Ω^n⟮E, F'⟯) (f : F →L[ℝ] F' →L[ℝ] F'') :
Ω^(m + n)⟮E, F''⟯ := fun e => ContinuousAlternatingMap.wedge_product (ω₁ e) (ω₂ e) f
Expand Down

0 comments on commit b92dabc

Please sign in to comment.