Skip to content

Commit 9fe5fb6

Browse files
author
LuuBluum
committed
Move imports around, clean up
1 parent 0888f6d commit 9fe5fb6

File tree

1 file changed

+1
-3
lines changed

1 file changed

+1
-3
lines changed

Cubical/Data/DiffInt/Base.agda

+1-3
Original file line numberDiff line numberDiff line change
@@ -4,11 +4,11 @@ module Cubical.Data.DiffInt.Base where
44
open import Cubical.Foundations.Prelude
55

66
open import Cubical.HITs.SetQuotients
7-
open import Cubical.HITs.SetQuotients.Properties
87
open import Cubical.Foundations.Isomorphism
98

109
open import Cubical.Data.Sigma
1110
open import Cubical.Data.Nat hiding (+-comm ; +-assoc) renaming (_+_ to _+ℕ_)
11+
open import Cubical.Data.Int
1212

1313
rel : (ℕ × ℕ) (ℕ × ℕ) Type₀
1414
rel (a₀ , b₀) (a₁ , b₁) = x ≡ y
@@ -21,8 +21,6 @@ rel (a₀ , b₀) (a₁ , b₁) = x ≡ y
2121

2222
-- Proof of equivalence between Int and DiffInt
2323

24-
open import Cubical.Data.Int
25-
2624
private
2725
-- Prove all the identities for ℕ×ℕ first and use that to build to ℤ
2826

0 commit comments

Comments
 (0)