Skip to content

Commit

Permalink
fix FPAlgebra
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Jun 8, 2024
1 parent 1f864a5 commit 11c6f4d
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion Cubical/Algebra/CommAlgebra/FPAlgebra/Base.agda
Original file line number Diff line number Diff line change
Expand Up @@ -51,7 +51,7 @@ module _ {R : CommRing ℓ} where
evPolyHomomorphic A B f P values =
(fst f) (evPoly A P values) ≡⟨ refl ⟩
(fst f) (fst (freeInducedHom A values) P) ≡⟨ refl ⟩
fst (f ∘a freeInducedHom A values) P ≡⟨ cong (λ u fst u P) (natIndHomR f values) ⟩
fst (f ∘a freeInducedHom A values) P ≡⟨ cong (λ u fst u P) (natIndHomR {A = A} {B = B} f values) ⟩
fst (freeInducedHom B (fst f ∘ values)) P ≡⟨ refl ⟩
evPoly B P (fst f ∘ values) ∎
where open AlgebraHoms
Expand Down
4 changes: 2 additions & 2 deletions Cubical/Algebra/CommAlgebra/FPAlgebra/Instances.agda
Original file line number Diff line number Diff line change
Expand Up @@ -78,13 +78,13 @@ module _ (R : CommRing ℓ) where
inverse1 : fromA ∘a toA ≡ idAlgebraHom _
inverse1 =
fromA ∘a toA
≡⟨ sym (unique _ _ _ _ _ _ (λ i cong (fst fromA) (
≡⟨ sym (unique _ _ B _ _ _ (λ i cong (fst fromA) (
fst toA (generator n emptyGen i)
≡⟨ inducedHomOnGenerators _ _ _ _ _ _ ⟩
Construction.var i
∎))) ⟩
inducedHom n emptyGen B (generator _ _) (relationsHold _ _)
≡⟨ unique _ _ _ _ _ _ (λ i refl) ⟩
≡⟨ unique _ _ B _ _ _ (λ i refl) ⟩
idAlgebraHom _
inverse2 : toA ∘a fromA ≡ idAlgebraHom _
Expand Down

0 comments on commit 11c6f4d

Please sign in to comment.