File tree Expand file tree Collapse file tree 1 file changed +2
-4
lines changed
Cubical/Algebra/CommAlgebra/FP Expand file tree Collapse file tree 1 file changed +2
-4
lines changed Original file line number Diff line number Diff line change 33module Cubical.Algebra.CommAlgebra.FP.Quotient where
44
55open import Cubical.Foundations.Prelude
6- open import Cubical.Foundations.Equiv
7- open import Cubical.Foundations.Isomorphism
86open import Cubical.Foundations.Function
97open import Cubical.Foundations.Structure
108
@@ -20,9 +18,9 @@ open import Cubical.Algebra.CommAlgebra.FGIdeal
2018open import Cubical.Algebra.CommAlgebra.FP
2119
2220private variable
23- ℓ ℓ' : Level
21+ ℓ : Level
2422
25- module _ {R : CommRing ℓ} {k : ℕ} (A : CommAlgebra R ℓ' ) (fpA : FPsOf R A) (G : FinVec ⟨ A ⟩ₐ k) where
23+ module _ {R : CommRing ℓ} {k : ℕ} (A : CommAlgebra R ℓ) (fpA : FPsOf R A) (G : FinVec ⟨ A ⟩ₐ k) where
2624 open FinitePresentation (fst fpA)
2725 ψ⁻¹ : CommAlgebraHom (A) fpAlg
2826 ψ⁻¹ = CommAlgebraEquiv→CommAlgebraHom (invCommAlgebraEquiv (snd fpA))
You can’t perform that action at this time.
0 commit comments