2014-12-15 21:43:42 +00:00
|
|
|
/-
|
|
|
|
Copyright (c) 2014 Microsoft Corporation. All rights reserved.
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
|
|
|
|
Module: init.sigma
|
|
|
|
Author: Leonardo de Moura, Jeremy Avigad, Floris van Doorn
|
|
|
|
-/
|
2014-12-01 04:34:12 +00:00
|
|
|
prelude
|
|
|
|
import init.num init.wf init.logic init.tactic
|
|
|
|
|
|
|
|
structure sigma {A : Type} (B : A → Type) :=
|
2014-12-20 02:23:08 +00:00
|
|
|
mk :: (pr1 : A) (pr2 : B pr1)
|
2014-12-01 04:34:12 +00:00
|
|
|
|
|
|
|
notation `Σ` binders `,` r:(scoped P, sigma P) := r
|
2014-11-17 04:08:52 +00:00
|
|
|
|
|
|
|
namespace sigma
|
2014-12-20 02:23:08 +00:00
|
|
|
notation `pr₁` := pr1
|
|
|
|
notation `pr₂` := pr2
|
|
|
|
notation `⟨`:max t:(foldr `,` (e r, mk e r)) `⟩`:0 := t --input ⟨ ⟩ as \< \>
|
2014-12-01 04:34:12 +00:00
|
|
|
|
|
|
|
namespace ops
|
2014-12-20 02:23:08 +00:00
|
|
|
postfix `.1`:(max+1) := pr1
|
|
|
|
postfix `.2`:(max+1) := pr2
|
2014-12-01 04:34:12 +00:00
|
|
|
end ops
|
|
|
|
|
2014-12-11 23:48:09 +00:00
|
|
|
open ops well_founded
|
2014-12-01 04:34:12 +00:00
|
|
|
|
2014-11-17 04:08:52 +00:00
|
|
|
section
|
|
|
|
variables {A : Type} {B : A → Type}
|
|
|
|
variable (Ra : A → A → Prop)
|
|
|
|
variable (Rb : ∀ a, B a → B a → Prop)
|
|
|
|
|
|
|
|
-- Lexicographical order based on Ra and Rb
|
|
|
|
inductive lex : sigma B → sigma B → Prop :=
|
2014-12-11 23:48:09 +00:00
|
|
|
left : ∀{a₁ b₁} a₂ b₂, Ra a₁ a₂ → lex ⟨a₁, b₁⟩ ⟨a₂, b₂⟩,
|
|
|
|
right : ∀a {b₁ b₂}, Rb a b₁ b₂ → lex ⟨a, b₁⟩ ⟨a, b₂⟩
|
2014-11-17 04:08:52 +00:00
|
|
|
end
|
|
|
|
|
|
|
|
context
|
|
|
|
parameters {A : Type} {B : A → Type}
|
|
|
|
parameters {Ra : A → A → Prop} {Rb : Π a : A, B a → B a → Prop}
|
|
|
|
infix `≺`:50 := lex Ra Rb
|
|
|
|
|
2014-12-11 23:48:09 +00:00
|
|
|
definition lex.accessible {a} (aca : acc Ra a) (acb : ∀a, well_founded (Rb a)) : ∀ (b : B a), acc (lex Ra Rb) ⟨a, b⟩ :=
|
2014-11-17 04:08:52 +00:00
|
|
|
acc.rec_on aca
|
2014-12-11 23:48:09 +00:00
|
|
|
(λxa aca (iHa : ∀y, Ra y xa → ∀b : B y, acc (lex Ra Rb) ⟨y, b⟩),
|
2014-11-17 04:08:52 +00:00
|
|
|
λb : B xa, acc.rec_on (acb xa b)
|
|
|
|
(λxb acb
|
2014-12-12 20:36:51 +00:00
|
|
|
(iHb : ∀ (y : B xa), Rb xa y xb → acc (lex Ra Rb) ⟨xa, y⟩),
|
2014-12-11 23:48:09 +00:00
|
|
|
acc.intro ⟨xa, xb⟩ (λp (lt : p ≺ ⟨xa, xb⟩),
|
2014-11-17 04:08:52 +00:00
|
|
|
have aux : xa = xa → xb == xb → acc (lex Ra Rb) p, from
|
2014-12-11 23:48:09 +00:00
|
|
|
@lex.rec_on A B Ra Rb (λp₁ p₂, p₂.1 = xa → p₂.2 == xb → acc (lex Ra Rb) p₁)
|
|
|
|
p ⟨xa, xb⟩ lt
|
2014-12-12 20:36:51 +00:00
|
|
|
(λ (a₁ : A) (b₁ : B a₁) (a₂ : A) (b₂ : B a₂) (H : Ra a₁ a₂) (eq₂ : a₂ = xa) (eq₃ : b₂ == xb),
|
|
|
|
begin cases eq₂, exact (iHa a₁ H b₁) end)
|
|
|
|
(λ (a : A) (b₁ b₂ : B a) (H : Rb a b₁ b₂) (eq₂ : a = xa) (eq₃ : b₂ == xb),
|
|
|
|
begin cases eq₂, cases eq₃, exact (iHb b₁ H) end),
|
2014-11-17 04:08:52 +00:00
|
|
|
aux rfl !heq.refl)))
|
|
|
|
|
|
|
|
-- The lexicographical order of well founded relations is well-founded
|
|
|
|
definition lex.wf (Ha : well_founded Ra) (Hb : ∀ x, well_founded (Rb x)) : well_founded (lex Ra Rb) :=
|
|
|
|
well_founded.intro (λp, destruct p (λa b, lex.accessible (Ha a) Hb b))
|
|
|
|
|
|
|
|
end
|
|
|
|
end sigma
|