File tree Expand file tree Collapse file tree 2 files changed +6
-6
lines changed
Expand file tree Collapse file tree 2 files changed +6
-6
lines changed Original file line number Diff line number Diff line change @@ -219,7 +219,7 @@ theorem containsThenInsertIfNew_snd [TransCmp cmp] (h : t.WF) {k : α} {v : β k
219219
220220@[simp, grind =]
221221theorem get?_emptyc [TransCmp cmp] [LawfulEqCmp cmp] {a : α} :
222- (∅ : DTreeMap α β cmp).get? a = none :=
222+ (∅ : Raw α β cmp).get? a = none :=
223223 Impl.get?_empty
224224
225225theorem get?_of_isEmpty [TransCmp cmp] [LawfulEqCmp cmp] (h : t.WF) {a : α} :
@@ -537,7 +537,7 @@ end Const
537537
538538@[simp, grind =]
539539theorem getD_emptyc [TransCmp cmp] [LawfulEqCmp cmp] {a : α} {fallback : β a} :
540- (∅ : DTreeMap α β cmp).getD a fallback = fallback :=
540+ (∅ : Raw α β cmp).getD a fallback = fallback :=
541541 Impl.getD_empty
542542
543543theorem getD_of_isEmpty [TransCmp cmp] [LawfulEqCmp cmp] (h : t.WF) {a : α} {fallback : β a} :
@@ -666,7 +666,7 @@ theorem getD_congr [TransCmp cmp] (h : t.WF) {a b : α} {fallback : β} (hab : c
666666end Const
667667
668668@[simp, grind =]
669- theorem getKey?_emptyc {a : α} : (∅ : DTreeMap α β cmp).getKey? a = none :=
669+ theorem getKey?_emptyc {a : α} : (∅ : Raw α β cmp).getKey? a = none :=
670670 Impl.getKey?_empty
671671
672672theorem getKey?_of_isEmpty [TransCmp cmp] (h : t.WF) {a : α} :
Original file line number Diff line number Diff line change @@ -204,7 +204,7 @@ theorem size_le_size_erase [TransCmp cmp] (h : t.WF) {k : α} :
204204 TreeMap.Raw.size_le_size_erase h
205205
206206@[simp, grind =]
207- theorem get?_emptyc {a : α} : (∅ : TreeSet α cmp).get? a = none :=
207+ theorem get?_emptyc {a : α} : (∅ : Raw α cmp).get? a = none :=
208208 TreeMap.Raw.getKey?_emptyc
209209
210210theorem get?_of_isEmpty [TransCmp cmp] (h : t.WF) {a : α} :
@@ -313,7 +313,7 @@ theorem get_eq [TransCmp cmp] [LawfulEqCmp cmp] (h : t.WF) {k : α} (h' : k ∈
313313
314314@[simp, grind =]
315315theorem get!_emptyc {a : α} [Inhabited α] :
316- (∅ : TreeSet α cmp).get! a = default :=
316+ (∅ : Raw α cmp).get! a = default :=
317317 TreeMap.Raw.getKey!_emptyc
318318
319319theorem get!_of_isEmpty [TransCmp cmp] [Inhabited α] (h : t.WF) {a : α} :
@@ -373,7 +373,7 @@ theorem get!_eq_of_mem [TransCmp cmp] [LawfulEqCmp cmp] [Inhabited α] (h : t.WF
373373
374374@[simp, grind =]
375375theorem getD_emptyc {a : α} {fallback : α} :
376- (∅ : TreeSet α cmp).getD a fallback = fallback :=
376+ (∅ : Raw α cmp).getD a fallback = fallback :=
377377 TreeMap.Raw.getKeyD_emptyc
378378
379379theorem getD_of_isEmpty [TransCmp cmp] (h : t.WF) {a fallback : α} :
You can’t perform that action at this time.
0 commit comments