Skip to content

Commit

Permalink
Move Rationals around
Browse files Browse the repository at this point in the history
  • Loading branch information
timorl committed Jul 18, 2023
1 parent b56db83 commit 2a510bc
Show file tree
Hide file tree
Showing 14 changed files with 33 additions and 33 deletions.
Original file line number Diff line number Diff line change
Expand Up @@ -4,12 +4,12 @@
-}
{-# OPTIONS --safe #-}
module Cubical.Algebra.CommRing.Instances.QuoQ where
module Cubical.Algebra.CommRing.Instances.Rationals where

open import Cubical.Foundations.Prelude

open import Cubical.Algebra.CommRing
open import Cubical.HITs.Rationals.QuoQ
open import Cubical.Data.Rationals
renaming (ℚ to ℚType ; _+_ to _+ℚ_; _·_ to _·ℚ_; -_ to -ℚ_)

open CommRingStr
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@
-}
{-# OPTIONS --safe #-}
module Cubical.Algebra.Field.Instances.QuoQ where
module Cubical.Algebra.Field.Instances.Rationals where

open import Cubical.Foundations.Prelude
open import Cubical.Foundations.HLevels
Expand All @@ -19,14 +19,14 @@ open import Cubical.Data.Int.MoreInts.QuoInt
; ·-zeroˡ to ·ℤ-zeroˡ
; ·-identityʳ to ·ℤ-identityʳ)
open import Cubical.HITs.SetQuotients as SetQuot
open import Cubical.HITs.Rationals.QuoQ
open import Cubical.Data.Rationals
using (ℚ ; ℕ₊₁→ℤ ; isEquivRel∼)

open import Cubical.Algebra.Field
open import Cubical.Algebra.CommRing
open import Cubical.Tactics.CommRingSolver.Reflection
open import Cubical.Algebra.CommRing.Instances.QuoInt
open import Cubical.Algebra.CommRing.Instances.QuoQ
open import Cubical.Algebra.CommRing.Instances.Rationals

open import Cubical.Relation.Nullary

Expand Down
7 changes: 7 additions & 0 deletions Cubical/Data/Rationals.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,7 @@
-- This is the preferred version of the rationals in the library. Other
-- versions can be found in the MoreRationals directory.
{-# OPTIONS --safe #-}
module Cubical.Data.Rationals where

open import Cubical.Data.Rationals.Base public
open import Cubical.Data.Rationals.Properties public
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
{-# OPTIONS --safe #-}
module Cubical.HITs.Rationals.QuoQ.Base where
module Cubical.Data.Rationals.Base where

open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Equiv
Expand Down
4 changes: 4 additions & 0 deletions Cubical/Data/Rationals/MoreRationals/HITQ.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,4 @@
{-# OPTIONS --safe #-}
module Cubical.Data.Rationals.MoreRationals.HITQ where

open import Cubical.Data.Rationals.MoreRationals.HITQ.Base public
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
{-# OPTIONS --safe #-}
module Cubical.HITs.Rationals.HITQ.Base where
module Cubical.Data.Rationals.MoreRationals.HITQ.Base where

open import Cubical.Foundations.Prelude
open import Cubical.Foundations.HLevels
Expand Down
6 changes: 6 additions & 0 deletions Cubical/Data/Rationals/MoreRationals/SigmaQ.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,6 @@
{-# OPTIONS --safe #-}
module Cubical.Data.Rationals.MoreRationals.SigmaQ where

open import Cubical.Data.Rationals.MoreRationals.SigmaQ.Base public

open import Cubical.Data.Rationals.MoreRationals.SigmaQ.Properties public
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
{-# OPTIONS --safe #-}
module Cubical.HITs.Rationals.SigmaQ.Base where
module Cubical.Data.Rationals.MoreRationals.SigmaQ.Base where

open import Cubical.Foundations.Prelude
open import Cubical.Foundations.HLevels
Expand Down
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
{-# OPTIONS --safe #-}
module Cubical.HITs.Rationals.SigmaQ.Properties where
module Cubical.Data.Rationals.MoreRationals.SigmaQ.Properties where

open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Function
Expand All @@ -17,8 +17,8 @@ open import Cubical.Data.Sigma
open import Cubical.Data.Nat.GCD
open import Cubical.Data.Nat.Coprime

open import Cubical.HITs.Rationals.QuoQ as Quo using (ℕ₊₁→ℤ)
import Cubical.HITs.Rationals.SigmaQ.Base as Sigma
open import Cubical.Data.Rationals as Quo using (ℕ₊₁→ℤ)
import Cubical.Data.Rationals.MoreRationals.SigmaQ.Base as Sigma


reduce : Quo.ℚ Sigma.ℚ
Expand Down
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
{-# OPTIONS --safe #-}
module Cubical.HITs.Rationals.QuoQ.Properties where
module Cubical.Data.Rationals.Properties where

open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Isomorphism
Expand All @@ -17,7 +17,7 @@ open import Cubical.Data.Sigma
open import Cubical.Data.Sum
open import Cubical.Relation.Nullary

open import Cubical.HITs.Rationals.QuoQ.Base
open import Cubical.Data.Rationals.Base

ℚ-cancelˡ : {a b} (c : ℕ₊₁) [ ℕ₊₁→ℤ c ℤ.· a / c ·₊₁ b ] ≡ [ a / b ]
ℚ-cancelˡ {a} {b} c = eq/ _ _
Expand Down
6 changes: 0 additions & 6 deletions Cubical/HITs/Rationals/HITQ.agda

This file was deleted.

6 changes: 0 additions & 6 deletions Cubical/HITs/Rationals/QuoQ.agda

This file was deleted.

6 changes: 0 additions & 6 deletions Cubical/HITs/Rationals/SigmaQ.agda

This file was deleted.

5 changes: 3 additions & 2 deletions Cubical/Papers/RepresentationIndependence.agda
Original file line number Diff line number Diff line change
Expand Up @@ -26,8 +26,9 @@ import Cubical.Data.Sigma.Properties as Sigma
import Cubical.HITs.PropositionalTruncation as PropositionalTruncation
import Cubical.HITs.Cost.Base as CostMonad
import Cubical.HITs.SetQuotients as SetQuotients
import Cubical.HITs.Rationals.QuoQ as SetQuoQ
import Cubical.HITs.Rationals.SigmaQ as SigmaQ
import Cubical.Data.Rationals as SetQuoQ
import Cubical.Data.Rationals.MoreRationals.SigmaQ
as SigmaQ
-- 3.1
import Cubical.Foundations.SIP as SIP
import Cubical.Structures.Axioms as Axioms
Expand Down

0 comments on commit 2a510bc

Please sign in to comment.