Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a8f6e23

Browse files
ChrisHughes24mergify[bot]
authored andcommitted
feat(data/list/basic): list.lex.not_nil_right (#1797)
1 parent 23e8ac7 commit a8f6e23

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

src/data/list/basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1573,6 +1573,8 @@ theorem cons_iff {r : α → α → Prop} [is_irrefl α r] {a l₁ l₂} :
15731573
lex r (a :: l₁) (a :: l₂) ↔ lex r l₁ l₂ :=
15741574
⟨λ h, by cases h with _ _ _ _ _ h _ _ _ _ h;
15751575
[exact h, exact (irrefl_of r a h).elim], lex.cons⟩
1576+
1577+
@[simp] theorem not_nil_right (r : α → α → Prop) (l : list α) : ¬ lex r l [].
15761578

15771579
instance is_order_connected (r : α → α → Prop)
15781580
[is_order_connected α r] [is_trichotomous α r] :

0 commit comments

Comments
 (0)