Skip to content

Commit

Permalink
chore(algebra/pi_tensor_product): Replace use of classical with decid…
Browse files Browse the repository at this point in the history
…able_eq (#5880)

This makes it consistent with `multilinear_map`, which also uses explicit decidability assumptions
  • Loading branch information
eric-wieser committed Jan 25, 2021
1 parent 1dfa81a commit 7188d80
Showing 1 changed file with 2 additions and 4 deletions.
6 changes: 2 additions & 4 deletions src/linear_algebra/pi_tensor_product.lean
Expand Up @@ -53,13 +53,11 @@ binary tensor product in `linear_algebra/tensor_product.lean`.
multilinear, tensor, tensor product
-/

noncomputable theory
open_locale classical
open function

section semiring

variables {ι : Type*} {R : Type*} [comm_semiring R]
variables {ι : Type*} [decidable_eq ι] {R : Type*} [comm_semiring R]
variables {R' : Type*} [comm_semiring R'] [algebra R' R]
variables {s : ι → Type*} [∀ i, add_comm_monoid (s i)] [∀ i, semimodule R (s i)]
variables {E : Type*} [add_comm_monoid E] [semimodule R E]
Expand Down Expand Up @@ -371,7 +369,7 @@ namespace pi_tensor_product
open pi_tensor_product
open_locale tensor_product

variables {ι : Type*} {R : Type*} [comm_ring R]
variables {ι : Type*} [decidable_eq ι] {R : Type*} [comm_ring R]
variables {s : ι → Type*} [∀ i, add_comm_group (s i)] [∀ i, module R (s i)]

/- Unlike for the binary tensor product, we require `R` to be a `comm_ring` here, otherwise
Expand Down

0 comments on commit 7188d80

Please sign in to comment.