Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 5bac21a

Browse files
committed
chore(algebra/module/pi): add pi.smul_def (#8311)
Sometimes it is useful to rewrite unapplied `s • x` (I need it in a branch that is not yet ready for review). We already have `pi.zero_def`, `pi.add_def`, etc.
1 parent 7fccf40 commit 5bac21a

File tree

1 file changed

+1
-0
lines changed

1 file changed

+1
-0
lines changed

src/algebra/module/pi.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -22,6 +22,7 @@ instance has_scalar {α : Type*} [Π i, has_scalar α $ f i] :
2222
has_scalar α (Π i : I, f i) :=
2323
⟨λ s x, λ i, s • (x i)⟩
2424

25+
lemma smul_def {α : Type*} [Π i, has_scalar α $ f i] (s : α) : s • x = λ i, s • x i := rfl
2526
@[simp] lemma smul_apply {α : Type*} [Π i, has_scalar α $ f i] (s : α) : (s • x) i = s • x i := rfl
2627

2728
instance has_scalar' {g : I → Type*} [Π i, has_scalar (f i) (g i)] :

0 commit comments

Comments
 (0)