Skip to content

Commit

Permalink
chore: cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
fgdorais committed Oct 25, 2024
1 parent 401211b commit 4e209ef
Showing 1 changed file with 0 additions and 9 deletions.
9 changes: 0 additions & 9 deletions Batteries/Data/Fin/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -84,15 +84,6 @@ protected def count (P : Fin n → Prop) [DecidablePred P] : Nat :=
/-- Find the first true value of a decidable predicate on `Fin n`, if there is one. -/
protected def find? (P : Fin n → Prop) [DecidablePred P] : Option (Fin n) :=
foldr n (fun i v => if P i then some i else v) none
-- match n, P, inst with
-- | 0, _, _ => none
-- | _+1, P, _ =>
-- if P 0 then
-- some 0
-- else
-- match Fin.find? fun i => P i.succ with
-- | some i => some i.succ
-- | none => none

/-- Custom recursor for `Fin (n+1)`. -/
def recZeroSuccOn {motive : Fin (n+1) → Sort _} (x : Fin (n+1))
Expand Down

0 comments on commit 4e209ef

Please sign in to comment.