Skip to content

Commit

Permalink
WIP: uniqueness
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Aug 31, 2022
1 parent 6461467 commit 688dce3
Showing 1 changed file with 29 additions and 2 deletions.
31 changes: 29 additions & 2 deletions Cubical/Algebra/CommAlgebra/UnivariatePolyList.agda
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,8 @@ module Cubical.Algebra.CommAlgebra.UnivariatePolyList where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Structure

open import Cubical.Data.Sigma

open import Cubical.Algebra.Ring
open import Cubical.Algebra.CommRing
open import Cubical.Algebra.AbGroup
Expand All @@ -17,7 +19,7 @@ private variable
ℓ ℓ' : Level

module _ (R : CommRing ℓ) where
open RingStr ⦃...⦄ -- Not CommRingStr, so it can be used in together with AlgebraStr
open RingStr ⦃...⦄ -- Not CommRingStr, so it can be used together with AlgebraStr
open PolyModTheory R
private
ListPoly = UnivariatePolyList R
Expand Down Expand Up @@ -182,7 +184,32 @@ module _ (R : CommRing ℓ) where
step8 : (r : ⟨ R ⟩) (p : _) _ ≡ _
step8 r p i = sym (⋆AssocL r 1a (inducedMap q)) i + (x · inducedMap p) · inducedMap q

open IsAlgebraHom
inducedHom : AlgebraHom (CommAlgebra→Algebra ListPolyCommAlgebra) A
fst inducedHom = inducedMap
snd inducedHom = makeIsAlgebraHom inducedMap1 inducedMap+ inducedMap· inducedMap⋆

{- Uniqueness -}
inducedHomUnique : (f : AlgebraHom (CommAlgebra→Algebra ListPolyCommAlgebra) A)
fst f X ≡ x
f ≡ inducedHom
inducedHomUnique f fX≡x =
Σ≡Prop
(λ _ isPropIsAlgebraHom _ _ _ _)
λ i p pwEq p i
where open IsAlgebraHom (snd f)
pwEq : (p : ⟨ ListPolyCommAlgebra ⟩) fst f p ≡ fst inducedHom p
pwEq =
ElimProp R
(λ p fst f p ≡ fst inducedHom p)
pres0
(λ r p IH
fst f (r ∷ p) ≡[ i ]⟨ fst f ((sym (+IdR r) i) ∷ p) ⟩
fst f ((r + 0r) ∷ p) ≡⟨ {!!}
fst f ([ r ] + (0r ∷ p)) ≡⟨ {!!}
fst f (r ⋆ 1a + X · p) ≡⟨ {!!}
fst f (r ⋆ 1a) + fst f (X · p) ≡⟨ {!!}
r ⋆ fst f 1a + fst f X · fst f p ≡⟨ {!!}
r ⋆ 1a + x · fst f p ≡[ i ]⟨ r ⋆ 1a + (x · IH i) ⟩
r ⋆ 1a + x · inducedMap p ≡⟨⟩
inducedMap (r ∷ p) ∎)
(is-set _ _)

0 comments on commit 688dce3

Please sign in to comment.