Skip to content

Commit a02a589

Browse files
committed
remove canonical mentions for now
1 parent 3f56141 commit a02a589

File tree

5 files changed

+2
-77
lines changed

5 files changed

+2
-77
lines changed

Mathlib/Tactic/Common.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -151,5 +151,3 @@ register_hint 200 omega
151151
register_hint 200 fun_prop
152152

153153
end Hint
154-
155-
-- example : True := by canonical +suggestions

Mathlib/Tactic/Linter/DirectoryDependency.lean

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -181,7 +181,6 @@ def allowedImportDirs : NamePrefixRel := .ofArray #[
181181
(`MathlibTest.Header, `Plausible),
182182
(`MathlibTest.Header, `ProofWidgets),
183183
(`MathlibTest.Header, `Qq),
184-
(`MathlibTest.Header, `Canonical),
185184
-- (`MathlibTest.Header, `Mathlib.Tactic),
186185
-- (`MathlibTest.Header, `Mathlib.Deprecated),
187186
(`MathlibTest.Header, `Batteries),
@@ -658,14 +657,13 @@ def directoryDependencyCheck (mainModule : Name) : CommandElabM (Array MessageDa
658657
else
659658
-- We always allow imports in the same directory (for each matching prefix),
660659
-- from `Init`, `Lean` and `Std`, as well as imports in `Aesop`, `Qq`, `Plausible`,
661-
-- `ImportGraph`, `ProofWidgets`, `LeanSearchClient` and `Canonical`
662-
-- (as these are imported in Tactic.Common).
660+
-- `ImportGraph`, `ProofWidgets` or `LeanSearchClient` (as these are imported in Tactic.Common).
663661
-- We also allow transitive imports of Mathlib.Init, as well as Mathlib.Init itself.
664662
let initImports := (← findImports ("Mathlib" / "Init.lean")).append
665663
#[`Mathlib.Init, `Mathlib.Tactic.DeclarationNames]
666664
let exclude := [
667665
`Init, `Std, `Lean,
668-
`Aesop, `Qq, `Plausible, `ImportGraph, `ProofWidgets, `LeanSearchClient, `Canonical
666+
`Aesop, `Qq, `Plausible, `ImportGraph, `ProofWidgets, `LeanSearchClient
669667
]
670668
let importsToCheck := imports.filter (fun imp ↦ !exclude.any (·.isPrefixOf imp))
671669
|>.filter (fun imp ↦ !matchingPrefixes.any (·.isPrefixOf imp))

Mathlib/Tactic/TacticAnalysis/Declarations.lean

Lines changed: 0 additions & 24 deletions
Original file line numberDiff line numberDiff line change
@@ -333,18 +333,6 @@ def tryAtEachStepAesop := tryAtEachStep
333333
fun _ _ => return ⟨TSyntax.raw <|
334334
mkNode `Aesop.Frontend.Parser.aesopTactic #[mkAtom "aesop", mkNullNode]⟩
335335

336-
-- /-- Run `canonical` at every step in proofs, reporting where it succeeds. -/
337-
-- register_option linter.tacticAnalysis.tryAtEachStepCanonical : Bool := {
338-
-- defValue := false
339-
-- }
340-
341-
-- @[tacticAnalysis linter.tacticAnalysis.tryAtEachStepCanonical,
342-
-- inherit_doc linter.tacticAnalysis.tryAtEachStepCanonical]
343-
-- def tryAtEachStepCanonical := tryAtEachStep
344-
-- -- As `canonical` isn't imported here, we construct the tactic syntax manually.
345-
-- fun _ _ => return ⟨TSyntax.raw <|
346-
-- mkNode `Mathlib.Tactic.Canonical.canonical #[mkAtom "canonical", mkNullNode]⟩
347-
348336
/-- Run `grind +suggestions` at every step in proofs, reporting where it succeeds. -/
349337
register_option linter.tacticAnalysis.tryAtEachStepGrindSuggestions : Bool := {
350338
defValue := false
@@ -365,18 +353,6 @@ register_option linter.tacticAnalysis.tryAtEachStepSimpAllSuggestions : Bool :=
365353
-- in `Logic/Equiv/Defs.lean` at `def cast` that I don't understand.
366354
def tryAtEachStepSimpAllSuggestions := tryAtEachStep fun _ _ => `(tactic| try simp_all? +suggestions)
367355

368-
-- /-- Run `canonical +suggestions` at every step in proofs, reporting where it succeeds. -/
369-
-- register_option linter.tacticAnalysis.tryAtEachStepCanonicalSuggestions : Bool := {
370-
-- defValue := false
371-
-- }
372-
373-
-- @[tacticAnalysis linter.tacticAnalysis.tryAtEachStepCanonicalSuggestions,
374-
-- inherit_doc linter.tacticAnalysis.tryAtEachStepSimpAllSuggestions]
375-
-- def tryAtEachStepCanonicalSuggestions := tryAtEachStep
376-
-- -- As `canonical` isn't imported here, we construct the tactic syntax manually.
377-
-- fun _ _ => return ⟨TSyntax.raw <|
378-
-- mkNode `Mathlib.Tactic.Canonical.canonical #[mkAtom "canonical", mkNullNode]⟩
379-
380356
-- TODO: add compatibility with `rintro` and `intros`
381357
/-- Suggest merging two adjacent `intro` tactics which don't pattern match. -/
382358
register_option linter.tacticAnalysis.introMerge : Bool := {

MathlibTest/canonical.lean

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

lakefile.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,6 @@ require "leanprover-community" / "proofwidgets" @ git "v0.0.83-pre2" -- ProofWid
1717
require "leanprover-community" / "importGraph" @ git "nightly-testing"
1818
require "leanprover-community" / "LeanSearchClient" @ git "nightly-testing"
1919
require "leanprover-community" / "plausible" @ git "nightly-testing"
20-
-- require "chasenorman" / "Canonical" @ git "nightly-2025-11-03"
2120

2221

2322
/-!

0 commit comments

Comments
 (0)