Zulip Chat Archive
Stream: general
Topic: universe resolutions
Kenny Lau (May 26 2020 at 14:05):
universes u v
variables {α : Type u} {β : Type v}
#check (ulift α = ulift β)
Kenny Lau (May 26 2020 at 14:05):
error:
type mismatch at application
ulift α = ulift β
term
ulift β
has type
Type (max v ?) : Type ((max v ?)+1)
but is expected to have type
Type (max u ?) : Type ((max u ?)+1)
Kenny Lau (May 26 2020 at 14:05):
is there a way to get Lean solve this automatically?
Kenny Lau (May 26 2020 at 14:05):
or is this generally undecidable?
Kenny Lau (May 26 2020 at 14:07):
lemma mk_range_eq_lift {α : Type u} {β : Type v} {f : α → β} (hf : injective f) :
lift.{v (max u w)} (# (range f)) = lift.{u (max v w)} (# α) :=
Reid Barton (May 26 2020 at 14:59):
Is this the solution (introduce an extra universe parameter) you want it to automatically find?
Last updated: Dec 20 2023 at 11:08 UTC