Skip to content

Commit

Permalink
fix: temporarily disable equation rendering
Browse files Browse the repository at this point in the history
  • Loading branch information
hargoniX committed Nov 18, 2023
1 parent b85fd6c commit 8c9e5cf
Showing 1 changed file with 7 additions and 1 deletion.
8 changes: 7 additions & 1 deletion DocGen4/Process/DefinitionInfo.lean
Original file line number Diff line number Diff line change
Expand Up @@ -36,8 +36,14 @@ def DefinitionInfo.ofDefinitionVal (v : DefinitionVal) : MetaM DefinitionInfo :=
let info ← Info.ofConstantVal v.toConstantVal
let isUnsafe := v.safety == DefinitionSafety.unsafe
let isNonComputable := isNoncomputable (← getEnv) v.name

try
let eqs? ← getEqnsFor? v.name
-- Temporary workaround until
-- https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/maxRecDepth.20in.20getEqnsFor.3F/near/402917295
-- is adddressed
let eqs? : Option (Array Name) := none
-- let eqs? ← getEqnsFor? v.name

match eqs? with
| some eqs =>
let equations ← eqs.mapM processEq
Expand Down

0 comments on commit 8c9e5cf

Please sign in to comment.