Skip to content

Commit

Permalink
deprecation
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 28, 2024
1 parent bcf14ad commit e205cfe
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Control/Random.lean
Original file line number Diff line number Diff line change
Expand Up @@ -93,7 +93,7 @@ def randBound (α : Type u)
(BoundedRandom.randomR lo hi h : RandGT g _ _)

def randFin {n : Nat} [RandomGen g] : RandGT g m (Fin n.succ) :=
fun ⟨g⟩ ↦ pure <| randNat g 0 n |>.map Fin.ofNat ULift.up
fun ⟨g⟩ ↦ pure <| randNat g 0 n |>.map (Fin.ofNat' _) ULift.up

instance {n : Nat} : Random m (Fin n.succ) where
random := randFin
Expand Down

0 comments on commit e205cfe

Please sign in to comment.