Skip to content

Commit

Permalink
chore: import plausible everywhere!
Browse files Browse the repository at this point in the history
  • Loading branch information
hargoniX committed Oct 28, 2024
1 parent 646e270 commit a2d68c4
Show file tree
Hide file tree
Showing 6 changed files with 6 additions and 4 deletions.
2 changes: 1 addition & 1 deletion .github/build.in.yml
Original file line number Diff line number Diff line change
Expand Up @@ -248,7 +248,7 @@ jobs:
- name: build everything
# make sure everything is available for test/import_all.lean
run: |
lake build Batteries Qq Aesop ProofWidgets
lake build Batteries Qq Aesop ProofWidgets Plausible
- name: test mathlib
id: test
Expand Down
2 changes: 1 addition & 1 deletion .github/workflows/bors.yml
Original file line number Diff line number Diff line change
Expand Up @@ -258,7 +258,7 @@ jobs:
- name: build everything
# make sure everything is available for test/import_all.lean
run: |
lake build Batteries Qq Aesop ProofWidgets
lake build Batteries Qq Aesop ProofWidgets Plausible
- name: test mathlib
id: test
Expand Down
2 changes: 1 addition & 1 deletion .github/workflows/build.yml
Original file line number Diff line number Diff line change
Expand Up @@ -265,7 +265,7 @@ jobs:
- name: build everything
# make sure everything is available for test/import_all.lean
run: |
lake build Batteries Qq Aesop ProofWidgets
lake build Batteries Qq Aesop ProofWidgets Plausible
- name: test mathlib
id: test
Expand Down
2 changes: 1 addition & 1 deletion .github/workflows/build_fork.yml
Original file line number Diff line number Diff line change
Expand Up @@ -262,7 +262,7 @@ jobs:
- name: build everything
# make sure everything is available for test/import_all.lean
run: |
lake build Batteries Qq Aesop ProofWidgets
lake build Batteries Qq Aesop ProofWidgets Plausible
- name: test mathlib
id: test
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Init.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,7 @@ import Mathlib.Tactic.Linter.OldObtain
import Mathlib.Tactic.Linter.RefineLinter
import Mathlib.Tactic.Linter.UnusedTactic
import Mathlib.Tactic.Linter.Style
import Plausible.Tactic -- allows everyone access to plausible

/-!
This is the root file in Mathlib: it is imported by virtually *all* Mathlib files.
Expand Down
1 change: 1 addition & 0 deletions test/import_all.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ import Batteries
import Aesop
import ProofWidgets
import Mathlib
import Plausible

/-!
Verify that Mathlib and all its upstream dependencies can be simultaneously imported.
Expand Down

0 comments on commit a2d68c4

Please sign in to comment.