xref: /XiangShan/src/main/scala/xiangshan/mem/lsqueue/LoadQueue.scala (revision 870f462d572cd0ef6bf86c91dcda5a5fab6e99d3)
1/***************************************************************************************
2* Copyright (c) 2020-2021 Institute of Computing Technology, Chinese Academy of Sciences
3* Copyright (c) 2020-2021 Peng Cheng Laboratory
4*
5* XiangShan is licensed under Mulan PSL v2.
6* You can use this software according to the terms and conditions of the Mulan PSL v2.
7* You may obtain a copy of Mulan PSL v2 at:
8*          http://license.coscl.org.cn/MulanPSL2
9*
10* THIS SOFTWARE IS PROVIDED ON AN "AS IS" BASIS, WITHOUT WARRANTIES OF ANY KIND,
11* EITHER EXPRESS OR IMPLIED, INCLUDING BUT NOT LIMITED TO NON-INFRINGEMENT,
12* MERCHANTABILITY OR FIT FOR A PARTICULAR PURPOSE.
13*
14* See the Mulan PSL v2 for more details.
15***************************************************************************************/
16
17package xiangshan.mem
18
19import chipsalliance.rocketchip.config.Parameters
20import chisel3._
21import chisel3.util._
22import utils._
23import utility._
24import xiangshan._
25import xiangshan.backend.fu.fpu.FPU
26import xiangshan.backend.rob.RobLsqIO
27import xiangshan.cache._
28import xiangshan.frontend.FtqPtr
29import xiangshan.ExceptionNO._
30import xiangshan.mem.mdp._
31import xiangshan.backend.Bundles.{DynInst, MemExuOutput, MemMicroOpRbExt}
32import xiangshan.backend.rob.RobPtr
33
34class LqPtr(implicit p: Parameters) extends CircularQueuePtr[LqPtr](
35  p => p(XSCoreParamsKey).VirtualLoadQueueSize
36){
37}
38
39object LqPtr {
40  def apply(f: Bool, v: UInt)(implicit p: Parameters): LqPtr = {
41    val ptr = Wire(new LqPtr)
42    ptr.flag := f
43    ptr.value := v
44    ptr
45  }
46}
47
48trait HasLoadHelper { this: XSModule =>
49  def rdataHelper(uop: DynInst, rdata: UInt): UInt = {
50    val fpWen = uop.fpWen
51    LookupTree(uop.fuOpType, List(
52      LSUOpType.lb   -> SignExt(rdata(7, 0) , XLEN),
53      LSUOpType.lh   -> SignExt(rdata(15, 0), XLEN),
54      /*
55          riscv-spec-20191213: 12.2 NaN Boxing of Narrower Values
56          Any operation that writes a narrower result to an f register must write
57          all 1s to the uppermost FLEN−n bits to yield a legal NaN-boxed value.
58      */
59      LSUOpType.lw   -> Mux(fpWen, FPU.box(rdata, FPU.S), SignExt(rdata(31, 0), XLEN)),
60      LSUOpType.ld   -> Mux(fpWen, FPU.box(rdata, FPU.D), SignExt(rdata(63, 0), XLEN)),
61      LSUOpType.lbu  -> ZeroExt(rdata(7, 0) , XLEN),
62      LSUOpType.lhu  -> ZeroExt(rdata(15, 0), XLEN),
63      LSUOpType.lwu  -> ZeroExt(rdata(31, 0), XLEN),
64    ))
65  }
66}
67
68class LqEnqIO(implicit p: Parameters) extends XSBundle {
69  private val LsExuCnt = backendParams.StaCnt + backendParams.LduCnt
70  val canAccept = Output(Bool())
71  val sqCanAccept = Input(Bool())
72  val needAlloc = Vec(LsExuCnt, Input(Bool()))
73  val req = Vec(LsExuCnt, Flipped(ValidIO(new DynInst)))
74  val resp = Vec(LsExuCnt, Output(new LqPtr))
75}
76
77class LqTriggerIO(implicit p: Parameters) extends XSBundle {
78  val hitLoadAddrTriggerHitVec = Input(Vec(3, Bool()))
79  val lqLoadAddrTriggerHitVec = Output(Vec(3, Bool()))
80}
81
82
83
84class LoadQueue(implicit p: Parameters) extends XSModule
85  with HasDCacheParameters
86  with HasCircularQueuePtrHelper
87  with HasLoadHelper
88  with HasPerfEvents
89{
90  val io = IO(new Bundle() {
91    val redirect = Flipped(Valid(new Redirect))
92    val enq = new LqEnqIO
93    val ldu = new Bundle() {
94        val stld_nuke_query = Vec(LoadPipelineWidth, Flipped(new LoadNukeQueryIO)) // from load_s2
95        val ldld_nuke_query = Vec(LoadPipelineWidth, Flipped(new LoadNukeQueryIO)) // from load_s2
96        val ldin         = Vec(LoadPipelineWidth, Flipped(Decoupled(new LqWriteBundle))) // from load_s3
97    }
98    val sta = new Bundle() {
99      val storeAddrIn = Vec(StorePipelineWidth, Flipped(Valid(new LsPipelineBundle))) // from store_s1
100    }
101    val std = new Bundle() {
102      val storeDataIn = Vec(StorePipelineWidth, Flipped(Valid(new MemExuOutput))) // from store_s0, store data, send to sq from rs
103    }
104    val sq = new Bundle() {
105      val stAddrReadySqPtr = Input(new SqPtr)
106      val stAddrReadyVec   = Input(Vec(StoreQueueSize, Bool()))
107      val stDataReadySqPtr = Input(new SqPtr)
108      val stDataReadyVec   = Input(Vec(StoreQueueSize, Bool()))
109      val stIssuePtr       = Input(new SqPtr)
110      val sqEmpty          = Input(Bool())
111    }
112    val ldout = Vec(LoadPipelineWidth, DecoupledIO(new MemExuOutput))
113    val ld_raw_data = Vec(LoadPipelineWidth, Output(new LoadDataFromLQBundle))
114    val replay = Vec(LoadPipelineWidth, Decoupled(new LsPipelineBundle))
115    val refill = Flipped(ValidIO(new Refill))
116    val tl_d_channel  = Input(new DcacheToLduForwardIO)
117    val release = Flipped(Valid(new Release))
118    val rollback = Output(Valid(new Redirect))
119    val rob = Flipped(new RobLsqIO)
120    val uncache = new UncacheWordIO
121    val trigger = Vec(LoadPipelineWidth, new LqTriggerIO)
122    val exceptionAddr = new ExceptionAddrIO
123    val lqFull = Output(Bool())
124    val lqDeq = Output(UInt(log2Up(CommitWidth + 1).W))
125    val lqCancelCnt = Output(UInt(log2Up(VirtualLoadQueueSize+1).W))
126    val lq_rep_full = Output(Bool())
127    val tlbReplayDelayCycleCtrl = Vec(4, Input(UInt(ReSelectLen.W)))
128    val l2_hint = Input(Valid(new L2ToL1Hint()))
129  })
130
131  val loadQueueRAR = Module(new LoadQueueRAR)  //  read-after-read violation
132  val loadQueueRAW = Module(new LoadQueueRAW)  //  read-after-write violation
133  val loadQueueReplay = Module(new LoadQueueReplay)  //  enqueue if need replay
134  val virtualLoadQueue = Module(new VirtualLoadQueue)  //  control state
135  val exceptionBuffer = Module(new LqExceptionBuffer) // exception buffer
136  val uncacheBuffer = Module(new UncacheBuffer) // uncache buffer
137
138  /**
139   * LoadQueueRAR
140   */
141  loadQueueRAR.io.redirect <> io.redirect
142  loadQueueRAR.io.release  <> io.release
143  loadQueueRAR.io.ldWbPtr  <> virtualLoadQueue.io.ldWbPtr
144  for (w <- 0 until LoadPipelineWidth) {
145    loadQueueRAR.io.query(w).req    <> io.ldu.ldld_nuke_query(w).req // from load_s1
146    loadQueueRAR.io.query(w).resp   <> io.ldu.ldld_nuke_query(w).resp // to load_s2
147    loadQueueRAR.io.query(w).revoke := io.ldu.ldld_nuke_query(w).revoke // from load_s3
148  }
149
150  /**
151   * LoadQueueRAW
152   */
153  loadQueueRAW.io.redirect         <> io.redirect
154  loadQueueRAW.io.storeIn          <> io.sta.storeAddrIn
155  loadQueueRAW.io.stAddrReadySqPtr <> io.sq.stAddrReadySqPtr
156  loadQueueRAW.io.stIssuePtr       <> io.sq.stIssuePtr
157  for (w <- 0 until LoadPipelineWidth) {
158    loadQueueRAW.io.query(w).req    <> io.ldu.stld_nuke_query(w).req // from load_s1
159    loadQueueRAW.io.query(w).resp   <> io.ldu.stld_nuke_query(w).resp // to load_s2
160    loadQueueRAW.io.query(w).revoke := io.ldu.stld_nuke_query(w).revoke // from load_s3
161  }
162
163  /**
164   * VirtualLoadQueue
165   */
166  virtualLoadQueue.io.redirect    <> io.redirect
167  virtualLoadQueue.io.enq         <> io.enq
168  virtualLoadQueue.io.ldin        <> io.ldu.ldin // from load_s3
169  virtualLoadQueue.io.lqFull      <> io.lqFull
170  virtualLoadQueue.io.lqDeq       <> io.lqDeq
171  virtualLoadQueue.io.lqCancelCnt <> io.lqCancelCnt
172
173  /**
174   * Load queue exception buffer
175   */
176  exceptionBuffer.io.redirect <> io.redirect
177  for ((buff, w) <- exceptionBuffer.io.req.zipWithIndex) {
178    buff.valid := io.ldu.ldin(w).valid // from load_s3
179    buff.bits := io.ldu.ldin(w).bits
180  }
181  io.exceptionAddr <> exceptionBuffer.io.exceptionAddr
182
183  /**
184   * Load uncache buffer
185   */
186  uncacheBuffer.io.redirect   <> io.redirect
187  uncacheBuffer.io.ldout      <> io.ldout
188  uncacheBuffer.io.ld_raw_data  <> io.ld_raw_data
189  uncacheBuffer.io.rob        <> io.rob
190  uncacheBuffer.io.uncache    <> io.uncache
191  uncacheBuffer.io.trigger    <> io.trigger
192  for ((buff, w) <- uncacheBuffer.io.req.zipWithIndex) {
193    buff.valid := io.ldu.ldin(w).valid // from load_s3
194    buff.bits := io.ldu.ldin(w).bits // from load_s3
195  }
196
197  // rollback
198  def selectOldest[T <: Redirect](valid: Seq[Bool], bits: Seq[T]): (Seq[Bool], Seq[T]) = {
199    assert(valid.length == bits.length)
200    if (valid.length == 0 || valid.length == 1) {
201      (valid, bits)
202    } else if (valid.length == 2) {
203      val res = Seq.fill(2)(Wire(ValidIO(chiselTypeOf(bits(0)))))
204      for (i <- res.indices) {
205        res(i).valid := valid(i)
206        res(i).bits := bits(i)
207      }
208      val oldest = Mux(valid(0) && valid(1), Mux(isAfter(bits(0).robIdx, bits(1).robIdx), res(1), res(0)), Mux(valid(0) && !valid(1), res(0), res(1)))
209      (Seq(oldest.valid), Seq(oldest.bits))
210    } else {
211      val left = selectOldest(valid.take(valid.length / 2), bits.take(bits.length / 2))
212      val right = selectOldest(valid.takeRight(valid.length - (valid.length / 2)), bits.takeRight(bits.length - (bits.length / 2)))
213      selectOldest(left._1 ++ right._1, left._2 ++ right._2)
214    }
215  }
216
217  val (rollbackSelV, rollbackSelBits) = selectOldest(
218                                          Seq(loadQueueRAW.io.rollback.valid, uncacheBuffer.io.rollback.valid),
219                                          Seq(loadQueueRAW.io.rollback.bits, uncacheBuffer.io.rollback.bits)
220                                        )
221  io.rollback.valid := rollbackSelV.head
222  io.rollback.bits := rollbackSelBits.head
223
224  /* <------- DANGEROUS: Don't change sequence here ! -------> */
225
226  /**
227   * LoadQueueReplay
228   */
229  loadQueueReplay.io.redirect         <> io.redirect
230  loadQueueReplay.io.enq              <> io.ldu.ldin // from load_s3
231  loadQueueReplay.io.storeAddrIn      <> io.sta.storeAddrIn // from store_s1
232  loadQueueReplay.io.storeDataIn      <> io.std.storeDataIn // from store_s0
233  loadQueueReplay.io.replay           <> io.replay
234  loadQueueReplay.io.refill           <> io.refill
235  loadQueueReplay.io.tl_d_channel     <> io.tl_d_channel
236  loadQueueReplay.io.stAddrReadySqPtr <> io.sq.stAddrReadySqPtr
237  loadQueueReplay.io.stAddrReadyVec   <> io.sq.stAddrReadyVec
238  loadQueueReplay.io.stDataReadySqPtr <> io.sq.stDataReadySqPtr
239  loadQueueReplay.io.stDataReadyVec   <> io.sq.stDataReadyVec
240  loadQueueReplay.io.sqEmpty          <> io.sq.sqEmpty
241  loadQueueReplay.io.lqFull           <> io.lq_rep_full
242  loadQueueReplay.io.ldWbPtr          <> virtualLoadQueue.io.ldWbPtr
243  loadQueueReplay.io.rarFull          <> loadQueueRAR.io.lqFull
244  loadQueueReplay.io.rawFull          <> loadQueueRAW.io.lqFull
245  loadQueueReplay.io.l2_hint          <> io.l2_hint
246  loadQueueReplay.io.tlbReplayDelayCycleCtrl <> io.tlbReplayDelayCycleCtrl
247
248  val full_mask = Cat(loadQueueRAR.io.lqFull, loadQueueRAW.io.lqFull, loadQueueReplay.io.lqFull)
249  XSPerfAccumulate("full_mask_000", full_mask === 0.U)
250  XSPerfAccumulate("full_mask_001", full_mask === 1.U)
251  XSPerfAccumulate("full_mask_010", full_mask === 2.U)
252  XSPerfAccumulate("full_mask_011", full_mask === 3.U)
253  XSPerfAccumulate("full_mask_100", full_mask === 4.U)
254  XSPerfAccumulate("full_mask_101", full_mask === 5.U)
255  XSPerfAccumulate("full_mask_110", full_mask === 6.U)
256  XSPerfAccumulate("full_mask_111", full_mask === 7.U)
257  XSPerfAccumulate("rollback", io.rollback.valid)
258
259  // perf cnt
260  val perfEvents = Seq(virtualLoadQueue, loadQueueRAR, loadQueueRAW, loadQueueReplay).flatMap(_.getPerfEvents) ++
261  Seq(
262    ("full_mask_000", full_mask === 0.U),
263    ("full_mask_001", full_mask === 1.U),
264    ("full_mask_010", full_mask === 2.U),
265    ("full_mask_011", full_mask === 3.U),
266    ("full_mask_100", full_mask === 4.U),
267    ("full_mask_101", full_mask === 5.U),
268    ("full_mask_110", full_mask === 6.U),
269    ("full_mask_111", full_mask === 7.U),
270    ("rollback", io.rollback.valid)
271  )
272  generatePerfEvent()
273  // end
274}