Skip to content

Commit

Permalink
MaxZX added
Browse files Browse the repository at this point in the history
  • Loading branch information
Franziskus Wiesnet committed Nov 12, 2024
1 parent 580e6a0 commit 92db749
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions Cubical/Algebra/MaxZX/PolynomialRingZnew.agda
Original file line number Diff line number Diff line change
@@ -1,8 +1,9 @@
{-# OPTIONS --cubical #-}

-- PolynomialRingZ.agda
module PolynomialRingZnew where
module Cubical.Algebra.MaxZX.PolynomialRingZnew where

open import Agda.Primitive
open import Agda.Primitive.Cubical
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Equiv
Expand All @@ -23,7 +24,7 @@ open import Cubical.Algebra.CommRing.Instances.Polynomials.UnivariatePolyList
open import Cubical.Data.Bool
open import Cubical.Data.Empty
open import Cubical.Tactics.CommRingSolver
open import ExplMaxIdeal
open import Cubical.Algebra.MaxZX.ExplMaxIdeal

{- record Inspect {A : Set} (x : A) : Set where
constructor what
Expand Down

0 comments on commit 92db749

Please sign in to comment.