bookshelf/common/Bookshelf/Tuple.lean

56 lines
1.4 KiB
Plaintext
Raw Normal View History

/-
# References
1. Enderton, Herbert B. A Mathematical Introduction to Logic. 2nd ed. San Diego:
Harcourt/Academic Press, 2001.
-/
import Mathlib.Tactic.Ring
universe u
/--[1]
An n-tuple is defined recursively as:
⟨x₁, ..., xₙ₊₁⟩ = ⟨⟨x₁, ..., xₙ⟩, xₙ₊₁⟩
2023-02-21 01:19:12 +00:00
TODO: As [1] notes, it is useful to define ⟨x⟩ = x. Is this syntactically
possible in Lean?
--/
2023-02-21 01:19:12 +00:00
inductive Tuple : (α : Type u) → Nat → Type u where
| only : α → Tuple α 1
| cons : {n : Nat} → Tuple α n → α → Tuple α (n + 1)
syntax (priority := high) "⟨" term,+ "⟩" : term
macro_rules
2023-02-21 01:19:12 +00:00
| `(⟨$x⟩) => `(Tuple.only $x)
| `(⟨$xs:term,*, $x⟩) => `(Tuple.cons ⟨$xs,*⟩ $x)
namespace Tuple
/--
Returns the value at the nth-index of the given tuple.
-/
def index (t : Tuple α n) (m : Nat) : 1 ≤ m ∧ m ≤ n → α := by
intro h
cases t
2023-02-21 01:19:12 +00:00
· case only last => exact last
. case cons n' init last =>
by_cases k : m = n' + 1
· exact last
· exact index init m (And.intro h.left (by
have h₂ : m + 1 ≤ n' + 1 := Nat.lt_of_le_of_ne h.right k
norm_num at h₂
exact h₂))
2023-02-21 01:19:12 +00:00
-- TODO: Prove `eq_by_index`.
-- TODO: Prove Lemma 0A [1].
theorem eq_by_index (t₁ t₂ : Tuple α n)
: (t₁ = t₂) ↔ (∀ i : Nat, 1 ≤ i ∧ i ≤ n → index t₁ i = index t₂ i) := by
apply Iff.intro
· sorry
· sorry
end Tuple