Skip to content

Commit

Permalink
Fix formatting
Browse files Browse the repository at this point in the history
  • Loading branch information
monsterkrampe committed Dec 11, 2024
1 parent cdc6b59 commit 0617166
Showing 1 changed file with 8 additions and 8 deletions.
16 changes: 8 additions & 8 deletions src/Std/Data/DHashMap/Internal/List/Associative.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2099,7 +2099,7 @@ theorem getKey?_insertList_of_mem [BEq α] [EquivBEq α]
{k k' : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Sigma.fst)) :
(mem : k ∈ toInsert.map Sigma.fst) :
getKey? k' (insertList l toInsert) = some k := by
rw [List.mem_map] at mem
rcases mem with ⟨pair, pair_mem, pair_eq⟩
Expand Down Expand Up @@ -2132,7 +2132,7 @@ theorem getKey_insertList_of_mem [BEq α] [EquivBEq α]
{k k' : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Sigma.fst))
(mem : k ∈ toInsert.map Sigma.fst)
{h} :
getKey k' (insertList l toInsert) h = k := by
rw [← Option.some_inj]
Expand All @@ -2157,7 +2157,7 @@ theorem getKey!_insertList_of_mem [BEq α] [EquivBEq α] [Inhabited α]
{k k' : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Sigma.fst)) :
(mem : k ∈ toInsert.map Sigma.fst) :
getKey! k' (insertList l toInsert) = k := by
rw [getKey!_eq_getKey?]
rw [getKey?_insertList_of_mem]
Expand All @@ -2181,7 +2181,7 @@ theorem getKeyD_insertList_of_mem [BEq α] [EquivBEq α]
{k k' fallback : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Sigma.fst)) :
(mem : k ∈ toInsert.map Sigma.fst) :
getKeyD k' (insertList l toInsert) fallback = k := by
rw [getKeyD_eq_getKey?]
rw [getKey?_insertList_of_mem]
Expand Down Expand Up @@ -2371,7 +2371,7 @@ theorem getKey?_insertListConst_of_mem [BEq α] [EquivBEq α]
{k k' : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Prod.fst)) :
(mem : k ∈ toInsert.map Prod.fst) :
getKey? k' (insertListConst l toInsert) = some k := by
unfold insertListConst
apply getKey?_insertList_of_mem
Expand All @@ -2398,7 +2398,7 @@ theorem getKey_insertListConst_of_mem [BEq α] [EquivBEq α]
{k k' : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Prod.fst))
(mem : k ∈ toInsert.map Prod.fst)
{h} :
getKey k' (insertListConst l toInsert) h = k := by
rw [← Option.some_inj]
Expand All @@ -2423,7 +2423,7 @@ theorem getKey!_insertListConst_of_mem [BEq α] [EquivBEq α] [Inhabited α]
{k k' : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Prod.fst)) :
(mem : k ∈ toInsert.map Prod.fst) :
getKey! k' (insertListConst l toInsert) = k := by
rw [getKey!_eq_getKey?]
rw [getKey?_insertListConst_of_mem]
Expand All @@ -2447,7 +2447,7 @@ theorem getKeyD_insertListConst_of_mem [BEq α] [EquivBEq α]
{k k' fallback : α} (k_beq : k == k')
(distinct_l : DistinctKeys l)
(distinct_toInsert : toInsert.Pairwise (fun a b => (a.1 == b.1) = false))
(mem : k ∈ (toInsert.map Prod.fst)) :
(mem : k ∈ toInsert.map Prod.fst) :
getKeyD k' (insertListConst l toInsert) fallback = k := by
rw [getKeyD_eq_getKey?]
rw [getKey?_insertListConst_of_mem]
Expand Down

0 comments on commit 0617166

Please sign in to comment.