import Mathlib.Tactic everywhere
This commit is contained in:
@@ -19,8 +19,14 @@ open Lean in
|
||||
modifyEnv (fun env => Lake.packageDepAttr.ext.addEntry env gameServerName)
|
||||
: Elab.Command.CommandElabM Unit)
|
||||
|
||||
-- require mathlib from git
|
||||
-- "https://github.com/leanprover-community/mathlib4" @ "88e129706828e01b7622d6635af1ca6667e25bac"
|
||||
|
||||
-- `Game` fix:
|
||||
require mathlib from git
|
||||
"https://github.com/leanprover-community/mathlib4" @ "88e129706828e01b7622d6635af1ca6667e25bac"
|
||||
"https://github.com/leanprover-community/mathlib4" @ "b04c509ef69fc7939b5f67715a635e15743dbe3c"
|
||||
|
||||
|
||||
|
||||
package Game where
|
||||
moreLeanArgs := #["-Dtactic.hygienic=false"]
|
||||
|
||||
Reference in New Issue
Block a user