@@ -5,8 +5,8 @@ inductive TEmpty : Type
55info: TEmpty : Type
66TEmpty.casesOn.{u} (motive : TEmpty → Sort u) (t : TEmpty) : motive t
77TEmpty.ctorIdx : TEmpty → Nat
8- TEmpty.noConfusion.{u} {P : Sort u} {x1 x2 : TEmpty} (h12 : x1 = x2 ) : TEmpty.noConfusionType P x1 x2
9- TEmpty.noConfusionType.{u} (P : Sort u) (x1 x2 : TEmpty) : Sort u
8+ TEmpty.noConfusion.{u} {P : Sort u} {t t' : TEmpty} (eq : t = t' ) : TEmpty.noConfusionType P t t'
9+ TEmpty.noConfusionType.{u} (P : Sort u) (t t' : TEmpty) : Sort u
1010TEmpty.rec.{u} (motive : TEmpty → Sort u) (t : TEmpty) : motive t
1111TEmpty.recOn.{u} (motive : TEmpty → Sort u) (t : TEmpty) : motive t
1212-/
@@ -58,11 +58,11 @@ TestStruct.mk.inj {foo bar foo✝ bar✝ : Int} :
5858 { foo := foo, bar := bar } = { foo := foo✝, bar := bar✝ } → foo = foo✝ ∧ bar = bar✝
5959TestStruct.mk.injEq (foo bar foo✝ bar✝ : Int) :
6060 ({ foo := foo, bar := bar } = { foo := foo✝, bar := bar✝ }) = (foo = foo✝ ∧ bar = bar✝)
61- TestStruct.mk.noConfusion.{u} ( P : Sort u) ( foo bar foo' bar' : Int)
62- (h : { foo := foo, bar := bar } = { foo := foo', bar := bar' }) (k : foo = foo' → bar = bar' → P) : P
61+ TestStruct.mk.noConfusion.{u} { P : Sort u} { foo bar foo' bar' : Int}
62+ (eq : { foo := foo, bar := bar } = { foo := foo', bar := bar' }) (k : foo = foo' → bar = bar' → P) : P
6363TestStruct.mk.sizeOf_spec (foo bar : Int) : sizeOf { foo := foo, bar := bar } = 1 + sizeOf foo + sizeOf bar
64- TestStruct.noConfusion.{u} {P : Sort u} {x1 x2 : TestStruct} (h12 : x1 = x2 ) : TestStruct.noConfusionType P x1 x2
65- TestStruct.noConfusionType.{u} (P : Sort u) (x1 x2 : TestStruct) : Sort u
64+ TestStruct.noConfusion.{u} {P : Sort u} {t t' : TestStruct} (eq : t = t' ) : TestStruct.noConfusionType P t t'
65+ TestStruct.noConfusionType.{u} (P : Sort u) (t t' : TestStruct) : Sort u
6666TestStruct.rec.{u} {motive : TestStruct → Sort u} (mk : (foo bar : Int) → motive { foo := foo, bar := bar })
6767 (t : TestStruct) : motive t
6868TestStruct.recOn.{u} {motive : TestStruct → Sort u} (t : TestStruct)
@@ -79,10 +79,10 @@ TestStruct.casesOn.{u} {motive : TestStruct → Sort u} (t : TestStruct)
7979TestStruct.ctorIdx : TestStruct → Nat
8080TestStruct.foo (self : TestStruct) : Int
8181TestStruct.mk (foo bar : Int) : TestStruct
82- TestStruct.mk.noConfusion.{u} ( P : Sort u) ( foo bar foo' bar' : Int)
83- (h : { foo := foo, bar := bar } = { foo := foo', bar := bar' }) (k : foo = foo' → bar = bar' → P) : P
84- TestStruct.noConfusion.{u} {P : Sort u} {x1 x2 : TestStruct} (h12 : x1 = x2 ) : TestStruct.noConfusionType P x1 x2
85- TestStruct.noConfusionType.{u} (P : Sort u) (x1 x2 : TestStruct) : Sort u
82+ TestStruct.mk.noConfusion.{u} { P : Sort u} { foo bar foo' bar' : Int}
83+ (eq : { foo := foo, bar := bar } = { foo := foo', bar := bar' }) (k : foo = foo' → bar = bar' → P) : P
84+ TestStruct.noConfusion.{u} {P : Sort u} {t t' : TestStruct} (eq : t = t' ) : TestStruct.noConfusionType P t t'
85+ TestStruct.noConfusionType.{u} (P : Sort u) (t t' : TestStruct) : Sort u
8686TestStruct.rec.{u} {motive : TestStruct → Sort u} (mk : (foo bar : Int) → motive { foo := foo, bar := bar })
8787 (t : TestStruct) : motive t
8888TestStruct.recOn.{u} {motive : TestStruct → Sort u} (t : TestStruct)
0 commit comments