-
Notifications
You must be signed in to change notification settings - Fork 295
[Merged by Bors] - chore(*): remove after the fact attribute [irreducible]
at several places
#18168
Changes from 15 commits
b77ebea
9850793
4f4b36e
40aeec5
96ed219
8d0736d
bdde0ff
a0a68db
52ff242
9c83044
ad19234
e2f74c1
dde45ea
1f3ebfa
ac23872
ecf7789
File filter
Filter by extension
Conversations
Jump to
Diff view
Diff view
There are no files selected for viewing
Original file line number | Diff line number | Diff line change |
---|---|---|
|
@@ -40,7 +40,10 @@ section involute | |
|
||
/-- Grade involution, inverting the sign of each basis vector. -/ | ||
def involute : clifford_algebra Q →ₐ[R] clifford_algebra Q := | ||
clifford_algebra.lift Q ⟨-(ι Q), λ m, by simp⟩ | ||
begin | ||
refine clifford_algebra.lift Q _, | ||
exact ⟨-(ι Q), λ m, by simp only [linear_map.neg_apply, mul_neg, neg_mul, ι_sq_scalar, neg_neg]⟩ | ||
end | ||
There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. Did squeezing the simp not work without the separate There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. It didn't work without the separate There was a problem hiding this comment. Choose a reason for hiding this commentThe reason will be displayed to describe this comment to others. Learn more. Thanks for trying! |
||
|
||
@[simp] lemma involute_ι (m : M) : involute (ι Q m) = -ι Q m := | ||
lift_ι_apply _ _ m | ||
|
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
This is pretty unfortunate: having
lift R f (ι R x) = f
true feels like havingsum.elim f g (sum.inl x) = f x
true definitionally, in that it's effectively the recursor for the type.This is expecially jarrying ater #18121, which only just introduced this defeq for
tensor_product
.What happens if we just don't make it irreducible at all?
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
In the current situation, iota is made irreducible a few lines below, so this lemma doesn't hold definitionally by the end of this file currently, and the PR doesn't change that.
We could also drop irreducibility of iota and lift, but I guess it was there for performance reasons. This would probably belong to a different PR, though.
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
Ah, good point. I still think this is unfortunate, but now agree that's out of scope for this PR