We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent c6f62d4 commit bc7a252Copy full SHA for bc7a252
Cubical/Algebra/CommRing/Instances/Polynomials/Typevariate/Base.agda
@@ -15,7 +15,7 @@ module Cubical.Algebra.CommRing.Instances.Polynomials.Typevariate.Base where
15
This file contains
16
* the definition of the free commutative algebra on a type I over a commutative ring R as a HIT
17
(let us call that R[I])
18
- * a prove that the construction is an commutative R-algebra
+ * the homomorphism R -> R[I], which turns this CommRing into a CommAlgebra
19
For more, see the Properties file.
20
-}
21
open import Cubical.Foundations.Prelude
0 commit comments