@@ -27,7 +27,7 @@ info: Vec.match_on_same_ctor.het.{u_1, u} {α : Type u} {motive : {a : Nat} →
2727/--
2828info: Vec.match_on_same_ctor.{u_1, u} {α : Type u}
2929 {motive : {a : Nat} → (t t_1 : Vec α a) → t.ctorIdx = t_1.ctorIdx → Sort u_1} {a✝ : Nat} (t t✝ : Vec α a✝)
30- (h : t.ctorIdx = t✝.ctorIdx) (nil : motive nil nil ⋯)
30+ (h : t.ctorIdx = t✝.ctorIdx) (nil : Unit → motive nil nil ⋯)
3131 (cons : (a : α) → {n : Nat} → (a_1 : Vec α n) → (a' : α) → (a'_1 : Vec α n) → motive (cons a a_1) (cons a' a'_1) ⋯) :
3232 motive t t✝ h
3333-/
@@ -54,10 +54,10 @@ info: Vec.match_on_same_ctor.splitter.{u_1, u} {α : Type u}
5454/--
5555info: Vec.match_on_same_ctor.eq_2.{u_1, u} {α : Type u}
5656 {motive : {a : Nat} → (t t_1 : Vec α a) → t.ctorIdx = t_1.ctorIdx → Sort u_1} (a✝ : α) (n : Nat) (a✝¹ : Vec α n)
57- (a'✝ : α) (a'✝¹ : Vec α n) (nil : motive nil nil ⋯)
57+ (a'✝ : α) (a'✝¹ : Vec α n) (nil : Unit → motive nil nil ⋯)
5858 (cons : (a : α) → {n : Nat} → (a_1 : Vec α n) → (a' : α) → (a'_1 : Vec α n) → motive (cons a a_1) (cons a' a'_1) ⋯) :
5959 (match n + 1, Vec.cons a✝ a✝¹, Vec.cons a'✝ a'✝¹ with
60- | 0, Vec.nil, Vec.nil, ⋯ => nil
60+ | 0, Vec.nil, Vec.nil, ⋯ => nil ()
6161 | n + 1, Vec.cons a a_1, Vec.cons a' a'_1, ⋯ => cons a a_1 a' a'_1) =
6262 cons a✝ a✝¹ a'✝ a'✝¹
6363-/
@@ -72,7 +72,7 @@ info: Vec.match_on_same_ctor.eq_2.{u_1, u} {α : Type u}
7272
7373def decEqVec {α} {a} [DecidableEq α] (x : @Vec α a) (x_1 : @Vec α a) : Decidable (x = x_1) :=
7474 if h : Vec.ctorIdx x = Vec.ctorIdx x_1 then
75- Vec.match_on_same_ctor x x_1 h (isTrue rfl)
75+ Vec.match_on_same_ctor x x_1 h (fun _ => isTrue rfl)
7676 @fun a_1 _ a_2 b b_1 =>
7777 if h_1 : @a_1 = @b then by
7878 subst h_1
@@ -137,7 +137,7 @@ run_meta mkCasesOnSameCtor `List.match_on_same_ctor ``List
137137
138138/--
139139info: List.match_on_same_ctor.{u_1, u} {α : Type u} {motive : (t t_1 : List α) → t.ctorIdx = t_1.ctorIdx → Sort u_1}
140- (t t✝ : List α) (h : t.ctorIdx = t✝.ctorIdx) (nil : motive [ ] [] ⋯)
140+ (t t✝ : List α) (h : t.ctorIdx = t✝.ctorIdx) (nil : Unit → motive [ ] [] ⋯)
141141 (cons : (head : α) → (tail : List α) → (head' : α) → (tail' : List α) → motive (head :: tail) (head' :: tail') ⋯) :
142142 motive t t✝ h
143143-/
0 commit comments