Skip to content

Commit afa49f1

Browse files
committed
oops
1 parent ca77768 commit afa49f1

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Std/Data/DTreeMap/Lemmas.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -28,7 +28,7 @@ private local instance : Coe (Type v) (α → Type v) where coe γ := fun _ =>
2828

2929
private theorem ext {t t' : DTreeMap α β cmp} : t.inner = t'.inner → t = t' := by
3030
cases t; cases t'; rintro rfl; rfl
31-
/-
31+
3232
@[simp]
3333
theorem isEmpty_emptyc : (∅ : DTreeMap α β cmp).isEmpty :=
3434
Impl.isEmpty_empty
@@ -4133,7 +4133,7 @@ theorem maxKeyD_alter_eq_self [TransCmp cmp] {k f}
41334133
end Const
41344134

41354135
end Max
4136-
-/
4136+
41374137
namespace Equiv
41384138

41394139
variable {t₁ t₂ t₃ : DTreeMap α β cmp} {δ : Type w} {m : Type w → Type w}

0 commit comments

Comments
 (0)