We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent ca77768 commit afa49f1Copy full SHA for afa49f1
src/Std/Data/DTreeMap/Lemmas.lean
@@ -28,7 +28,7 @@ private local instance : Coe (Type v) (α → Type v) where coe γ := fun _ =>
28
29
private theorem ext {t t' : DTreeMap α β cmp} : t.inner = t'.inner → t = t' := by
30
cases t; cases t'; rintro rfl; rfl
31
-/-
+
32
@[simp]
33
theorem isEmpty_emptyc : (∅ : DTreeMap α β cmp).isEmpty :=
34
Impl.isEmpty_empty
@@ -4133,7 +4133,7 @@ theorem maxKeyD_alter_eq_self [TransCmp cmp] {k f}
4133
end Const
4134
4135
end Max
4136
--/
4137
namespace Equiv
4138
4139
variable {t₁ t₂ t₃ : DTreeMap α β cmp} {δ : Type w} {m : Type w → Type w}
0 commit comments