Skip to content

Algebra.Solver.Ring allows us to specify a coefficient ring, but not here #2700

Open
@onestruggler

Description

@onestruggler

This line fixed the coefficient ring to be the target ring:

homo : Homomorphism ℓ₁ ℓ₂ ℓ₁ ℓ₂

It seems that it should be in some file like "Algebra.Solver.Ring.Simple".

Probably due to this, it seems that I cannot use "Tactic.RingSolver" on abstract rings since I cannot provide an "AlmostCommutativeRing" (from an abstract ring), which requires a field "0≟_ : (x : Carrier) → Maybe (0# ≈ x)". I cannot do pattern matching on "#0", or in general on elements of an abstract ring.

The paper "Proving Equalities in a Commutative Ring Done Right in Coq" says their mothod works for abstract rings in paper's abstract. Algebra.Solver.Ring seems to work for abstract rings, but I haven't checked this yet.

Metadata

Metadata

Assignees

No one assigned

    Labels

    Type

    No type

    Projects

    No projects

    Milestone

    No milestone

    Relationships

    None yet

    Development

    No branches or pull requests

    Issue actions