File tree Expand file tree Collapse file tree 2 files changed +4
-7
lines changed
Data/Iterators/Combinators/Monadic Expand file tree Collapse file tree 2 files changed +4
-7
lines changed Original file line number Diff line number Diff line change @@ -1360,13 +1360,6 @@ theorem Relation.TransGen.trans {α : Sort u} {r : α → α → Prop} {a b c} :
13601360 | single h => exact TransGen.tail hab h
13611361 | tail _ h ih => exact TransGen.tail ih h
13621362
1363- theorem Relation.TransGen.mono {α : Sort u} {r s : α → α → Prop } (h : ∀ a b, r a b → s a b) {a b} :
1364- TransGen r a b → TransGen s a b := by
1365- intro hab
1366- induction hab
1367- case single rab => exact .single (h _ _ rab)
1368- case tail rbc ih => exact .tail ih (h _ _ rbc)
1369-
13701363/-! # Subtype -/
13711364
13721365namespace Subtype
Original file line number Diff line number Diff line change @@ -34,6 +34,10 @@ structure Take (α : Type w) (m : Type w → Type w') {β : Type w} [Iterator α
3434 countdown : Nat
3535 /-- Internal implementation detail of the iterator library -/
3636 inner : IterM (α := α) m β
37+ /--
38+ Internal implementation detail of the iterator library.
39+ This proof term ensures that a `take` always produces a finite iterator from a productive one.
40+ -/
3741 finite : countdown > 0 ∨ Finite α m
3842
3943/--
You can’t perform that action at this time.
0 commit comments