Skip to content

Commit

Permalink
chore(*): fix authorship for split files (#4480)
Browse files Browse the repository at this point in the history
A few files with missing copyright headers in #4477 came from splitting up older files, so the attribution was incorrect:
- `data/setoid/partition.lean` was split from `data/setoid.lean` in #2853.
- `data/finset/order.lean` was split from `algebra/big_operators.lean` in #3495.
- `group_theory/submonoid/operations.lean` was split from `group_theory/submonoid.lean` in  #3058.
  • Loading branch information
bryangingechen authored and adomani committed Oct 7, 2020
1 parent 54389b7 commit 103b05a
Show file tree
Hide file tree
Showing 3 changed files with 11 additions and 6 deletions.
8 changes: 6 additions & 2 deletions src/data/finset/order.lean
Original file line number Diff line number Diff line change
@@ -1,11 +1,15 @@
/-
Copyright (c) 2020 Scott Morrison. All rights reserved.
Copyright (c) 2018 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
Authors: Mario Carneiro, Kenny Lau
-/

import data.finset.basic

/-!
# Finsets of ordered types
-/

universes u v w
variables {α : Type u}

Expand Down
4 changes: 2 additions & 2 deletions src/data/setoid/partition.lean
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
/-
Copyright (c) 2020 Yury G. Kudryashov. All rights reserved.
Copyright (c) 2019 Amelia Livingston. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury G. Kudryashov
Authors: Amelia Livingston, Bryan Gin-ge Chen
-/

import data.setoid.basic
Expand Down
5 changes: 3 additions & 2 deletions src/group_theory/submonoid/operations.lean
Original file line number Diff line number Diff line change
@@ -1,7 +1,8 @@
/-
Copyright (c) 2020 Yury G. Kudryashov. All rights reserved.
Copyright (c) 2018 Johannes Hölzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury G. Kudryashov
Authors: Johannes Hölzl, Kenny Lau, Johan Commelin, Mario Carneiro, Kevin Buzzard,
Amelia Livingston, Yury Kudryashov
-/

import group_theory.submonoid.basic
Expand Down

0 comments on commit 103b05a

Please sign in to comment.