Skip to content

Commit

Permalink
use mathlib
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed May 18, 2024
1 parent e65326c commit 7a039e1
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions scripts/count_decls.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2024 Kyle Miller. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kyle Miller, Damiano Testa
-/
import Mathlib.Data.Nat.Defs
import Mathlib --.Data.Nat.Defs

/-!
# `count_decls` -- a tally of declarations in `Mathlib`
Expand Down Expand Up @@ -80,6 +80,6 @@ elab "count_decls" : command => do
logInfo m!"{s.types.toArray}"
-- logInfo s!"Theorems {s.thms}\nData {s.data}\nPredicates {s.preds}\nTypes {s.types}"

count_decls
--count_decls

end PeriodicReports

0 comments on commit 7a039e1

Please sign in to comment.