Skip to content

Commit

Permalink
delete LiftLets
Browse files Browse the repository at this point in the history
  • Loading branch information
kmill committed Dec 21, 2024
1 parent 17c25ae commit ba4c611
Show file tree
Hide file tree
Showing 6 changed files with 0 additions and 246 deletions.
1 change: 0 additions & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4816,7 +4816,6 @@ import Mathlib.Tactic.IntervalCases
import Mathlib.Tactic.IrreducibleDef
import Mathlib.Tactic.Lemma
import Mathlib.Tactic.Lift
import Mathlib.Tactic.LiftLets
import Mathlib.Tactic.Linarith
import Mathlib.Tactic.Linarith.Datatypes
import Mathlib.Tactic.Linarith.Frontend
Expand Down
1 change: 0 additions & 1 deletion Mathlib/LinearAlgebra/CliffordAlgebra/EvenEquiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ Authors: Eric Wieser
import Mathlib.LinearAlgebra.CliffordAlgebra.Conjugation
import Mathlib.LinearAlgebra.CliffordAlgebra.Even
import Mathlib.LinearAlgebra.QuadraticForm.Prod
import Mathlib.Tactic.LiftLets

/-!
# Isomorphisms with the even subalgebra of a Clifford algebra
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -117,7 +117,6 @@ import Mathlib.Tactic.IntervalCases
import Mathlib.Tactic.IrreducibleDef
import Mathlib.Tactic.Lemma
import Mathlib.Tactic.Lift
import Mathlib.Tactic.LiftLets
import Mathlib.Tactic.Linarith
import Mathlib.Tactic.Linarith.Datatypes
import Mathlib.Tactic.Linarith.Frontend
Expand Down
134 changes: 0 additions & 134 deletions Mathlib/Tactic/LiftLets.lean

This file was deleted.

108 changes: 0 additions & 108 deletions MathlibTest/LiftLets.lean

This file was deleted.

1 change: 0 additions & 1 deletion scripts/noshake.json
Original file line number Diff line number Diff line change
Expand Up @@ -115,7 +115,6 @@
"Mathlib.Tactic.Lemma",
"Mathlib.Tactic.LibrarySearch",
"Mathlib.Tactic.Lift",
"Mathlib.Tactic.LiftLets",
"Mathlib.Tactic.Linarith",
"Mathlib.Tactic.Linarith.Frontend",
"Mathlib.Tactic.Linarith.Lemmas",
Expand Down

0 comments on commit ba4c611

Please sign in to comment.