Skip to content

Commit 91c0406

Browse files
committed
chore: Remove Init.CCLemmas (#10696)
Those lemmas were weird and unused, except the last few about transitivity of `=` and `≠`, which I moved to `Logic.Basic`
1 parent 719d6e1 commit 91c0406

File tree

8 files changed

+10
-136
lines changed

8 files changed

+10
-136
lines changed

Mathlib.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2364,7 +2364,6 @@ import Mathlib.GroupTheory.Transfer
23642364
import Mathlib.InformationTheory.Hamming
23652365
import Mathlib.Init.Algebra.Classes
23662366
import Mathlib.Init.Align
2367-
import Mathlib.Init.CCLemmas
23682367
import Mathlib.Init.Classes.Order
23692368
import Mathlib.Init.Classical
23702369
import Mathlib.Init.Control.Combinators

Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2020 Kevin Kappelmann. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Kevin Kappelmann
55
-/
6-
import Mathlib.Init.CCLemmas
76
import Mathlib.Algebra.ContinuedFractions.Computation.Basic
87
import Mathlib.Algebra.ContinuedFractions.Translations
98

Mathlib/Algebra/Group/Pi/Lemmas.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Simon Hudon, Patrick Massot
55
-/
6-
import Mathlib.Init.CCLemmas
76
import Mathlib.Algebra.Group.Hom.Instances
87
import Mathlib.Data.Set.Function
98
import Mathlib.Logic.Pairwise

Mathlib/Algebra/Ring/Equiv.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2018 Johannes Hölzl. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov
55
-/
6-
import Mathlib.Init.CCLemmas
76
import Mathlib.Algebra.Field.IsField
87
import Mathlib.Algebra.Group.Equiv.Basic
98
import Mathlib.Algebra.Group.Opposite

Mathlib/Data/Finset/Card.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2015 Microsoft Corporation. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Leonardo de Moura, Jeremy Avigad
55
-/
6-
import Mathlib.Init.CCLemmas
76
import Mathlib.Data.Finset.Image
87

98
#align_import data.finset.card from "leanprover-community/mathlib"@"65a1391a0106c9204fe45bc73a039f056558cb83"

Mathlib/Data/List/BigOperators/Lemmas.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -3,17 +3,16 @@ Copyright (c) 2017 Johannes Hölzl. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl, Floris van Doorn, Sébastien Gouëzel, Alex J. Best
55
-/
6-
import Mathlib.Init.CCLemmas
7-
import Mathlib.Data.List.BigOperators.Basic
86
import Mathlib.Algebra.Group.Opposite
97
import Mathlib.Algebra.GroupPower.Basic
108
import Mathlib.Algebra.GroupWithZero.Commute
119
import Mathlib.Algebra.GroupWithZero.Divisibility
1210
import Mathlib.Algebra.Order.Monoid.OrderDual
1311
import Mathlib.Algebra.Ring.Basic
14-
import Mathlib.Algebra.Ring.Divisibility.Basic
1512
import Mathlib.Algebra.Ring.Commute
13+
import Mathlib.Algebra.Ring.Divisibility.Basic
1614
import Mathlib.Data.Int.Units
15+
import Mathlib.Data.List.BigOperators.Basic
1716

1817
#align_import data.list.big_operators.lemmas from "leanprover-community/mathlib"@"f694c7dead66f5d4c80f446c796a5aad14707f0e"
1918

Mathlib/Init/CCLemmas.lean

Lines changed: 0 additions & 128 deletions
This file was deleted.

Mathlib/Logic/Basic.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -529,6 +529,14 @@ theorem ball_mem_comm {α β} [Membership α β] {s : β} {p : α → α → Pro
529529

530530
#align ne_of_apply_ne ne_of_apply_ne
531531

532+
lemma ne_of_eq_of_ne (h₁ : a = b) (h₂ : b ≠ c) : a ≠ c := h₁.symm ▸ h₂
533+
lemma ne_of_ne_of_eq (h₁ : a ≠ b) (h₂ : b = c) : a ≠ c := h₂ ▸ h₁
534+
535+
alias Eq.trans_ne := ne_of_eq_of_ne
536+
alias Ne.trans_eq := ne_of_ne_of_eq
537+
#align eq.trans_ne Eq.trans_ne
538+
#align ne.trans_eq Ne.trans_eq
539+
532540
theorem eq_equivalence : Equivalence (@Eq α) :=
533541
⟨Eq.refl, @Eq.symm _, @Eq.trans _⟩
534542
#align eq_equivalence eq_equivalence

0 commit comments

Comments
 (0)