We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 24dd4ca commit a3e910dCopy full SHA for a3e910d
Cache/Requests.lean
@@ -241,7 +241,7 @@ def getRemoteRepo (mathlibDepPath : FilePath) : IO RepoInfo := do
241
return {repo := repo, useFirst := false}
242
243
-- FRO cache may be flaky: https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/The.20cache.20doesn't.20work/near/411058849
244
-def useFROCache : Bool := true
+def useFROCache : Bool := false
245
246
/-- Public URL for mathlib cache -/
247
def URL : String :=
0 commit comments