Skip to content

Commit

Permalink
split(algebra/hom/ring): Split off algebra.ring.basic (#14144)
Browse files Browse the repository at this point in the history
Move `non_unital_ring_hom` and `ring_hom` to a new file `algebra.hom.ring`.

Crediting
* Amelia for #1305
* Jireh for #13430
  • Loading branch information
YaelDillies committed May 17, 2022
1 parent 4ae5e7a commit 65bf134
Show file tree
Hide file tree
Showing 8 changed files with 558 additions and 563 deletions.
2 changes: 1 addition & 1 deletion src/algebra/field/basic.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2014 Robert Lewis. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Robert Lewis, Leonardo de Moura, Johannes Hölzl, Mario Carneiro
-/
import algebra.ring.basic
import algebra.hom.ring

/-!
# Fields and division rings
Expand Down
3 changes: 1 addition & 2 deletions src/algebra/group_power/basic.lean
Expand Up @@ -3,9 +3,8 @@ Copyright (c) 2015 Jeremy Avigad. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jeremy Avigad, Robert Y. Lewis
-/
import algebra.hom.ring
import data.nat.basic
import tactic.monotonicity.basic
import group_theory.group_action.defs

/-!
# Power operations on monoids and groups
Expand Down

0 comments on commit 65bf134

Please sign in to comment.