Skip to content

Commit 8a59faf

Browse files
Saransh-cppandreasabel
authored andcommitted
Final Data.Product import simplifications (#2052)
1 parent 35f151a commit 8a59faf

File tree

143 files changed

+131
-148
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

143 files changed

+131
-148
lines changed

README/Case.agda

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,6 @@ module README.Case where
1212
open import Data.Fin hiding (pred)
1313
open import Data.Maybe hiding (from-just)
1414
open import Data.Nat hiding (pred)
15-
open import Data.Product
1615
open import Function.Base using (case_of_; case_return_of_)
1716
open import Relation.Nullary
1817
open import Relation.Binary

README/Data/Container/Indexed.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@ module README.Data.Container.Indexed where
1111
open import Data.Unit
1212
open import Data.Empty
1313
open import Data.Nat.Base
14-
open import Data.Product
14+
open import Data.Product.Base using (_,_)
1515
open import Function.Base using (_∋_)
1616
open import Data.W.Indexed
1717
open import Data.Container.Indexed

README/Data/Integer.agda

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -51,7 +51,6 @@ ex₅ i j = ℤₚ.*-comm i j
5151
-- provides some combinators for equational reasoning.
5252

5353
open P.≡-Reasoning
54-
open import Data.Product
5554

5655
ex₆ : i j i * (j + + 0) ≡ j * i
5756
ex₆ i j = begin

README/Data/List/Fresh.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ open import Data.Nat
1212
open import Data.List.Base
1313
open import Data.List.Fresh
1414
open import Data.List.Relation.Unary.AllPairs as AllPairs using (AllPairs)
15-
open import Data.Product
15+
open import Data.Product.Base using (_,_; proj₁; proj₂)
1616
open import Relation.Nary using (⌊_⌋; fromWitness)
1717

1818
-- A sorted list of natural numbers can be seen as a fresh list

README/Data/Record.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@
1111

1212
module README.Data.Record where
1313

14-
open import Data.Product
14+
open import Data.Product.Base using (_,_)
1515
open import Data.String
1616
open import Function.Base using (flip)
1717
open import Level

README/Data/Trie/NonDependent.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -56,7 +56,7 @@ import Data.Char.Properties as Char
5656
open import Data.List.Base as List using (List; []; _∷_)
5757
open import Data.List.Fresh as List# using (List#; []; _∷#_)
5858
open import Data.Maybe as Maybe
59-
open import Data.Product as Prod
59+
open import Data.Product.Base as Prod using (_×_; ∃; proj₁; _,_)
6060
open import Data.String.Base as String using (String)
6161
open import Data.String.Properties as String using (_≟_)
6262
open import Data.These as These

README/Data/Wrap.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ open import Data.Wrap
1313
open import Algebra
1414
open import Data.Nat
1515
open import Data.Nat.Properties
16-
open import Data.Product
16+
open import Data.Product.Base using (_,_; ∃; ∃₂; _×_)
1717
open import Level using (Level)
1818
open import Relation.Binary
1919

README/Design/Decidability.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ open import Data.List.Base using (List; []; _∷_)
1313
open import Data.List.Properties using (∷-injective)
1414
open import Data.Nat
1515
open import Data.Nat.Properties using (suc-injective)
16-
open import Data.Product
16+
open import Data.Product.Base using (uncurry)
1717
open import Data.Unit
1818
open import Function.Base using (id; _∘_)
1919
open import Relation.Binary.PropositionalEquality

README/Foreign/Haskell.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -22,7 +22,7 @@ open import Data.Bool.Base using (Bool; if_then_else_)
2222
open import Data.Char as Char
2323
open import Data.List.Base as List using (List; _∷_; []; takeWhile; dropWhile)
2424
open import Data.Maybe.Base using (Maybe; just; nothing)
25-
open import Data.Product
25+
open import Data.Product.Base using (_×_; _,_)
2626
open import Function
2727
open import Relation.Nullary.Decidable
2828

README/Inspect.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -14,7 +14,7 @@ module README.Inspect where
1414

1515
open import Data.Nat.Base
1616
open import Data.Nat.Properties
17-
open import Data.Product
17+
open import Data.Product.Base using (_×_; _,_)
1818
open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl)
1919
open import Relation.Binary.PropositionalEquality using (inspect)
2020

0 commit comments

Comments
 (0)