Skip to content

Commit

Permalink
polynomial ring is fp
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Aug 30, 2024
1 parent 9ce0eff commit 12dedb4
Show file tree
Hide file tree
Showing 3 changed files with 21 additions and 9 deletions.
4 changes: 2 additions & 2 deletions Cubical/Algebra/CommAlgebra/FGIdeal.agda
Original file line number Diff line number Diff line change
Expand Up @@ -33,5 +33,5 @@ syntax generatedIdeal A V = ⟨ V ⟩[ A ]
module _ {R : CommRing ℓ} (A : CommAlgebra R ℓ) where
open CommRingStr (A .fst .snd)

0FGIdeal : {n : ℕ} ⟨ replicateFinVec n 0r ⟩[ A ] ≡ (0Ideal R A)
0FGIdeal = 0FGIdealCommRing (CommAlgebra→CommRing A)
0FGIdeal≡0Ideal : {n : ℕ} ⟨ replicateFinVec n 0r ⟩[ A ] ≡ (0Ideal R A)
0FGIdeal≡0Ideal = 0FGIdealCommRing (CommAlgebra→CommRing A)
5 changes: 2 additions & 3 deletions Cubical/Algebra/CommAlgebra/FP/Base.agda
Original file line number Diff line number Diff line change
Expand Up @@ -27,9 +27,8 @@ private
ℓ ℓ' : Level

module _ (R : CommRing ℓ) where
abstract
Polynomials : (n : ℕ) CommAlgebra R ℓ
Polynomials n = R [ Fin n ]ₐ
Polynomials : (n : ℕ) CommAlgebra R ℓ
Polynomials n = R [ Fin n ]ₐ

FPCAlgebra : {m : ℕ} (n : ℕ) (relations : FinVec ⟨ Polynomials n ⟩ₐ m) CommAlgebra R ℓ
FPCAlgebra n relations = Polynomials n / ⟨ relations ⟩[ Polynomials n ]
Expand Down
21 changes: 17 additions & 4 deletions Cubical/Algebra/CommAlgebra/FP/Instances.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@
* R/⟨x₁,...,xₙ⟩ = R[⊥]/⟨x₁,...,xₙ⟩
* R/⟨x⟩ (as special case of the above)
-}
{-# OPTIONS --safe #-}
{-# OPTIONS --safe --lossy-unification #-}
module Cubical.Algebra.CommAlgebra.FP.Instances where

open import Cubical.Foundations.Prelude
Expand All @@ -30,7 +30,7 @@ open import Cubical.Algebra.CommRing.FGIdeal using (inclOfFGIdeal)
open import Cubical.Algebra.CommAlgebra
open import Cubical.Algebra.CommAlgebra.Instances.Polynomials
open import Cubical.Algebra.CommAlgebra.QuotientAlgebra
open import Cubical.Algebra.CommAlgebra.Ideal using (IdealsIn)
open import Cubical.Algebra.CommAlgebra.Ideal using (IdealsIn; 0Ideal)
open import Cubical.Algebra.CommAlgebra.FGIdeal
-- open import Cubical.Algebra.CommAlgebra.Instances.Initial
open import Cubical.Algebra.CommAlgebra.Instances.Unit
Expand All @@ -44,18 +44,31 @@ private

module _ (R : CommRing ℓ) where
open FinitePresentation
{-

module _ (n : ℕ) where
private
abstract
p : 0Ideal R (Polynomials R n) ≡ ⟨ emptyFinVec ⟨ Polynomials R n ⟩ₐ ⟩[ _ ]
p = sym $ 0FGIdeal≡0Ideal (Polynomials R n)

compute :
CommAlgebraEquiv (Polynomials R n) $ (Polynomials R n) / ⟨ emptyFinVec ⟨ Polynomials R n ⟩ₐ ⟩[ _ ]
compute =
transport (λ i CommAlgebraEquiv (Polynomials R n) ((Polynomials R n) / (p i))) $
zeroIdealQuotient (Polynomials R n)

polynomialsFP : FinitePresentation R (Polynomials R n)
polynomialsFP =
record {
n = n ;
m = 0 ;
relations = emptyFinVec ⟨ Polynomials R n ⟩ₐ ;
equiv = invCommAlgebraEquiv {!zeroIdealQuotient!}
equiv = invCommAlgebraEquiv compute
}

{-
{- Every (multivariate) polynomial algebra is finitely presented -}
module _ (n : ℕ) where
private
Expand Down

0 comments on commit 12dedb4

Please sign in to comment.