@@ -35,7 +35,7 @@ public theorem toList_ric {α : Type u} {β : Type v} (cmp : α → α → Order
3535 [TransCmp cmp] {t : Raw α β cmp} {wf : t.WF} {bound : α} :
3636 t[*...=bound].toList = t.toList.filter (fun e => (cmp e.fst bound).isLE) := by
3737 apply @DTreeMap.Internal.Const.toList_ric _ _ ⟨cmp⟩ _ _
38- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
38+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
3939
4040public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
4141 Rio.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RioSlice α β ⟨cmp⟩) :=
@@ -45,7 +45,7 @@ public theorem toList_rio {α : Type u} {β : Type v} (cmp : α → α → Order
4545 [TransCmp cmp] {t : Raw α β cmp} {wf : t.WF} {bound : α} :
4646 t[*...<bound].toList = t.toList.filter (fun e => (cmp e.fst bound).isLT) := by
4747 apply @DTreeMap.Internal.Const.toList_rio _ _ ⟨cmp⟩ _ _
48- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
48+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
4949
5050public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
5151 Rci.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RciSlice α β ⟨cmp⟩) :=
@@ -55,7 +55,7 @@ public theorem toList_rci {α : Type u} {β : Type v} (cmp : α → α → Order
5555 [TransCmp cmp] {t : Raw α β cmp} {wf : t.WF} {bound : α} :
5656 t[bound...*].toList = t.toList.filter (fun e => (cmp e.fst bound).isGE) := by
5757 apply @DTreeMap.Internal.Const.toList_rci _ _ ⟨cmp⟩ _ _
58- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
58+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
5959
6060public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
6161 Rco.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RcoSlice α β ⟨cmp⟩) :=
@@ -66,7 +66,7 @@ public theorem toList_rco {α : Type u} {β : Type v} (cmp : α → α → Order
6666 t[lowerBound...<upperBound].toList =
6767 t.toList.filter (fun e => (cmp e.fst lowerBound).isGE ∧ (cmp e.fst upperBound).isLT) := by
6868 apply @DTreeMap.Internal.Const.toList_rco _ _ ⟨cmp⟩ _ _
69- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
69+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
7070
7171public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
7272 Rcc.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RccSlice α β ⟨cmp⟩) :=
@@ -77,7 +77,7 @@ public theorem toList_rcc {α : Type u} {β : Type v} (cmp : α → α → Order
7777 t[lowerBound...=upperBound].toList =
7878 t.toList.filter (fun e => (cmp e.fst lowerBound).isGE ∧ (cmp e.fst upperBound).isLE) := by
7979 apply @DTreeMap.Internal.Const.toList_rcc _ _ ⟨cmp⟩ _ _
80- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
80+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
8181
8282public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
8383 Roi.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RoiSlice α β ⟨cmp⟩) :=
@@ -87,7 +87,7 @@ public theorem toList_roi {α : Type u} {β : Type v} (cmp : α → α → Order
8787 [TransCmp cmp] {t : Raw α β cmp} {wf : t.WF} {bound: α} : t[bound<...*].toList =
8888 t.toList.filter (fun e => (cmp e.fst bound).isGT) := by
8989 apply @DTreeMap.Internal.Const.toList_roi _ _ ⟨cmp⟩ _
90- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
90+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
9191
9292public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
9393 Roc.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RocSlice α β ⟨cmp⟩) :=
@@ -98,7 +98,7 @@ public theorem toList_roc {α : Type u} {β : Type v} (cmp : α → α → Order
9898 t[lowerBound<...=upperBound].toList =
9999 t.toList.filter (fun e => (cmp e.fst lowerBound).isGT ∧ (cmp e.fst upperBound).isLE) := by
100100 apply @DTreeMap.Internal.Const.toList_roc _ _ ⟨cmp⟩ _
101- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
101+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
102102
103103public instance {α : Type u} {β : Type v} (cmp : α → α → Ordering := by exact compare) :
104104 Roo.Sliceable (Raw α β cmp) α (@DTreeMap.Internal.Const.RooSlice α β ⟨cmp⟩) :=
@@ -109,6 +109,6 @@ public theorem toList_roo {α : Type u} {β : Type v} (cmp : α → α → Order
109109 t[lowerBound<...upperBound].toList =
110110 t.toList.filter (fun e => (cmp e.fst lowerBound).isGT ∧ (cmp e.fst upperBound).isLT) := by
111111 apply @DTreeMap.Internal.Const.toList_roo _ _ ⟨cmp⟩ _
112- . exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
112+ · exact @wf.out.out.ordered _ _ ⟨cmp⟩ _
113113
114114end Std.TreeMap.Raw
0 commit comments