You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
/path/to/Issue.agda:10,1-83
specializeType should never fail! This is a bug!
Error:
TC doesn't provide which error to catch
As discussed in person, I have a recursive type which depends on Pointwise, and defining the Pointwise instance manually doesn't help with deriving the Show instance for the original type. I tried to minimise the code as much as I could, but the example is still a bit complicated:
moduleIssuewhereopen importData.List.Relation.Binary.Pointwise.Baseusing (Pointwise)
open importData.List.Baseopen importAgda.Builtin.Sigmaopen importRelation.Binary.Coreusing (REL)
open importAgda.Primitiveusing (Level)
open importTactic.Derive.Showopen importTactic.Defaultsopen importClass.Show.CoredataAST (X :Set) :Setwhereconstr : (xs : List (AST X)) → AST X
Relation = { X :Set } → AST X → AST X →Set₁dataTranslation (R : Relation) { X :Set } : AST X → AST X →Set₁where
pointwiseCase
: {xs xs' : List (AST X)}
→ Pointwise (Translation R) xs xs'
→ Translation R (constr xs) (constr xs')
instance
Show-Pointwise
: {a : Level} {A :Set a} {b : Level} {B :Set b} {l : Level}
{xs : List A} {ys : List B} {r : REL A B l}
→ Show (Pointwise r xs ys)
Show-Pointwise = mkShow (λ x →"TODO")
unquoteDecl Show-Translation = derive-Show ((quote Translation , Show-Translation) ∷ [])
This throws the same error:
/path/to/Issue.agda:32,1-89
specializeType should never fail! This is a bug!
Error:
TC doesn't provide which error to catch
The text was updated successfully, but these errors were encountered:
The following code throws an error when compiling:
The error is:
As discussed in person, I have a recursive type which depends on
Pointwise
, and defining thePointwise
instance manually doesn't help with deriving theShow
instance for the original type. I tried to minimise the code as much as I could, but the example is still a bit complicated:This throws the same error:
The text was updated successfully, but these errors were encountered: