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

[Merged by Bors] - feat(ring_theory/ideal/operations): add an instance #6717

Closed
wants to merge 8 commits into from

Conversation

riccardobrasca
Copy link
Member

This instance has been suggested by @eric-wieser in #6640.

On my machine I get a deterministic timeout in ring_theory/finiteness at line 325, but in principle it seems a useful instance to have.

@@ -1235,6 +1235,12 @@ by simp only [ring_hom.algebra_map_to_algebra, ring_hom.comp_id]
instance {I : ideal A} : is_scalar_tower R A (ideal.quotient I) :=
is_scalar_tower.of_algebra_map_eq' (quotient.alg_map_eq R I)

instance quotient.is_scalar_tower' [algebra S A] [algebra S R] [is_scalar_tower S R A]
Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I think this one subsumes the instance above, so the one above can be removed. I doubt that will fix the timeout though.

Thanks for making the PR

Copy link
Member Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Indeed it doesn't...

If we want to keep this just for the record, should I close the PR?

Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I'll have a play with this tomorrow, now that you have a cache ready for me!

@eric-wieser eric-wieser added not-ready-to-merge WIP Work in progress and removed awaiting-review The author would like community review of the PR labels Mar 16, 2021
@bryangingechen bryangingechen changed the title feat(ring_theory/ideal/operations.lean): add an instance feat(ring_theory/ideal/operations): add an instance Mar 17, 2021
@riccardobrasca
Copy link
Member Author

@eric-wieser should I close this or do you want to work on it?

@eric-wieser
Copy link
Member

Well, I got CI passing on this (the failure was just a long line); I just haven't decided if it's actually a good idea.

@riccardobrasca
Copy link
Member Author

I can very well be wrong, but it seems to me a good instance to have.

@riccardobrasca riccardobrasca added awaiting-review The author would like community review of the PR and removed WIP Work in progress not-ready-to-merge labels Mar 23, 2021
@eric-wieser
Copy link
Member

Oh nice, I hadn't realized that this enabled more golfing.

Copy link
Collaborator

@Vierkantor Vierkantor left a comment

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I think this is a useful instance, since the corresponding algebra S I.quotient instance is already there. So I'll go ahead and merge this.

bors r+

@github-actions github-actions bot added ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) and removed awaiting-review The author would like community review of the PR labels Mar 26, 2021
bors bot pushed a commit that referenced this pull request Mar 26, 2021
This instance has been suggested by @eric-wieser in #6640.

On my machine I get a deterministic timeout in `ring_theory/finiteness` at line 325, but in principle it seems a useful instance to have. 

Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
@bors
Copy link

bors bot commented Mar 26, 2021

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(ring_theory/ideal/operations): add an instance [Merged by Bors] - feat(ring_theory/ideal/operations): add an instance Mar 26, 2021
@bors bors bot closed this Mar 26, 2021
@bors bors bot deleted the alg_quot branch March 26, 2021 14:24
b-mehta pushed a commit that referenced this pull request Apr 2, 2021
This instance has been suggested by @eric-wieser in #6640.

On my machine I get a deterministic timeout in `ring_theory/finiteness` at line 325, but in principle it seems a useful instance to have. 

Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

3 participants