Skip to content

Commit

Permalink
WIP
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Jul 24, 2024
1 parent cf402df commit efc76c4
Showing 1 changed file with 19 additions and 13 deletions.
32 changes: 19 additions & 13 deletions Cubical/Algebra/CommAlgebra/FreeCommAlgebra/OnCoproduct.agda
Original file line number Diff line number Diff line change
Expand Up @@ -13,9 +13,8 @@ open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Equiv
open import Cubical.Foundations.Equiv.BiInvertible
open import Cubical.Foundations.Isomorphism
open import Cubical.Foundations.Structure
open import Cubical.Foundations.Structure using (⟨_⟩; str)
open import Cubical.Foundations.GroupoidLaws
open import Cubical.Foundations.Structure

open import Cubical.Data.Sum as ⊎
open import Cubical.Data.Sigma
Expand Down Expand Up @@ -62,22 +61,29 @@ module CalculateFreeCommAlgebraOnCoproduct (R : CommRing ℓ) (I J : Type ℓ) w
_ = CommAlgebraHom R[I⊎J] (baseChange baseRingHom A)

inducedHomOverR : CommAlgebraHom R[I⊎J] AOverR
inducedHomOverR = inducedHom AOverR (rec (λ i var i ⋆ 1a) φ)
inducedHomOverR = inducedHom AOverR (⊎.rec (λ i var i ⋆ 1a) φ)

inducedHomOverR[I] : CommAlgebraHom R[I⊎J]overR[I] A
inducedHomOverR[I] = fst inducedHomOverR , record
{ pres0 = {!!}
; pres1 = {!!}
; pres+ = {!!}
; pres· = {!!}
; pres- = {!!}
; pres⋆ = {!!}
}
fst inducedHomOverR[I] = fst inducedHomOverR
snd inducedHomOverR[I] = record
{ pres0 = homStr .pres0
; pres1 = homStr .pres1
; pres+ = homStr .pres+
; pres· = homStr .pres·
; pres- = homStr .pres-
; pres⋆ = λ r x f (r ⋆ x) ≡⟨ {!!}
r ⋆ f x ∎
}
where open IsAlgebraHom
homStr = inducedHomOverR .snd
f = inducedHomOverR .fst
instance
_ = R[I⊎J]overR[I] .snd
_ = A .snd

-- (r : R[I]) → (y : R[I⊎J]) → f (r ⋆ 1a) ≡ r ⋆ 1a
-- (r : R[I]) → (y : R[I⊎J]) → f (var (inl i)) ≡ var i ⋆ 1a


{-
{-
We start by defining R[I][J] and R[I⊎J] as R[I] algebras,
Expand Down Expand Up @@ -310,4 +316,4 @@ module _ {R : CommRing ℓ} {I J : Type ℓ} where
invr-rightInv asBiInv = toFromOverR[I]
invl asBiInv = fst from
invl-leftInv asBiInv = fromTo
-}
-- -}

0 comments on commit efc76c4

Please sign in to comment.