Skip to content

Commit 25a2051

Browse files
wkrozowskidatokrat
andauthored
Update src/Std/Data/DTreeMap/Internal/Operations.lean
Co-authored-by: Paul Reichert <[email protected]>
1 parent ecf687b commit 25a2051

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Std/Data/DTreeMap/Internal/Operations.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -518,7 +518,7 @@ abbrev IteratedSlowNewInsertionInto [Ord α] (t) :=
518518
{ t' // ∀ {P : Impl α β → Prop}, P t → (∀ t'' a b, P t'' → P (t''.insertIfNew! a b)) → P t' }
519519

520520
/--
521-
Computes the union of the given tree maps. If a key appears in both maps, the entry contains in the second argument will appear in the result.
521+
Computes the union of the given tree maps. If a key appears in both maps, the entry contained in the second argument will appear in the result.
522522
523523
This function always merges the smaller map into the larger map.
524524
-/

0 commit comments

Comments
 (0)