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
-- set_option trace.elaborator_detail truedefmy_eq {A : Type*} (a b : A) : Prop := true
lemmaid_map_is_right_neutral {A : Type} (map : A -> A) :
my_eq (function.comp.{11 _} map map) map :=
sorry
with the error
kernel failed to type check declaration 'id_map_is_right_neutral' this is usually due to a buggy tactic or a bug in the builtin elaborator
elaborated type:
∀ {A : Type} (map : A → A), my_eq (map ∘ map) map
elaborated value:
λ {A : Type} (map : A → A), sorry
nested exception message:
type mismatch at application
@my_eq (A → A)
term
A → A
has type
Type
but is expected to have type
Type u_1
The following fails
with the error
It works if the
_
is replaced by1
.It seems like the elaborator has taken a wrong turn somewhere, by not unifying
u_1
with1
.See https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/HoTT3.20universe.20errors
The text was updated successfully, but these errors were encountered: