Skip to content

Commit

Permalink
chore(algebra/order/monoid): split into smaller files (#16861)
Browse files Browse the repository at this point in the history
This, along later PRs for `algebra.order.group` and `algebra.order.ring`, will replace #16792.

- [x] depends on: #16172

[![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)


Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
  • Loading branch information
semorrison and YaelDillies committed Oct 9, 2022
1 parent 4fc47d5 commit 8ef4f3f
Show file tree
Hide file tree
Showing 20 changed files with 1,625 additions and 1,467 deletions.
Expand Up @@ -5,7 +5,7 @@ Authors: Damiano Testa
-/
import data.zmod.basic
import ring_theory.subsemiring.basic
import algebra.order.monoid
import algebra.order.monoid.basic
/-!
A `canonically_ordered_comm_semiring` with two different elements `a` and `b` such that
Expand Down
2 changes: 1 addition & 1 deletion counterexamples/linear_order_with_pos_mul_pos_eq_zero.lean
Expand Up @@ -4,7 +4,7 @@ All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johan Commelin, Damiano Testa, Kevin Buzzard
-/
import algebra.order.monoid
import algebra.order.monoid.basic

/-!
An example of a `linear_ordered_comm_monoid_with_zero` in which the product of two positive
Expand Down
4 changes: 4 additions & 0 deletions src/algebra/order/group.lean
Expand Up @@ -5,6 +5,10 @@ Authors: Jeremy Avigad, Leonardo de Moura, Mario Carneiro, Johannes Hölzl
-/
import algebra.abs
import algebra.order.sub
import algebra.order.monoid.min_max
import algebra.order.monoid.prod
import algebra.order.monoid.type_tags
import algebra.order.monoid.units

/-!
# Ordered groups
Expand Down

0 comments on commit 8ef4f3f

Please sign in to comment.