leanprover-community / mathport

Mathport is a tool for porting Lean3 projects to Lean4
Apache License 2.0
41 stars 15 forks source link

Accidentally recursive definitions #168

Open gebner opened 2 years ago

gebner commented 2 years ago

Synport:

namespace Bool

theorem coe_sort_tt : coeSort.{1, 1} true = True :=
  coe_sort_tt

In Lean 3 coe_sort_tt would resolve to _root_.coe_sort_tt resulting in a non-recursive alias definition. But in Lean 4, coe_sort_tt now resolves to Bool.coe_sort_tt and we get a (nonterminating) recursive definition.