From 9ba47208278f7deea0dabed40a72fff89ecc5720 Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Fri, 1 Mar 2019 20:05:00 +0100 Subject: change id precedence --- Eq.thy | 26 +++++++++++++------------- 1 file changed, 13 insertions(+), 13 deletions(-) (limited to 'Eq.thy') diff --git a/Eq.thy b/Eq.thy index c6394dc..8814c1f 100644 --- a/Eq.thy +++ b/Eq.thy @@ -380,15 +380,15 @@ section \Transport\ schematic_goal transport: assumes [intro]: - "A: U i" "P: A \ U j" + "P: A \ U j" "A: U i" "x: A" "y: A" "p: x =[A] y" shows "?prf: P`x \ P`y" proof (path_ind' x y p) - show "\x. x: A \ id(P`x): P`x \ P`x" by derive + show "\x. x: A \ id P`x: P`x \ P`x" by derive qed routine definition transport :: "[t, t, t, t] \ t" ("(2transport[_, _, _] _)" [0, 0, 0, 1000]) -where "transport[P, x, y] p \ indEq (\a b. & (P`a \ P`b)) (\x. id (P`x)) x y p" +where "transport[P, x, y] p \ indEq (\a b. & (P`a \ P`b)) (\x. id P`x) x y p" syntax "_transport'" :: "[t, t] \ t" ("(2_*)" [1000]) @@ -405,13 +405,13 @@ end \ corollary transport_type: - assumes "A: U i" "P: A \ U j" "x: A" "y: A" "p: x =[A] y" + assumes "P: A \ U j" "A: U i" "x: A" "y: A" "p: x =[A] y" shows "transport[P, x, y] p: P`x \ P`y" unfolding transport_def using assms by (rule transport) lemma transport_comp: assumes [intro]: "A: U i" "P: A \ U j" "a: A" - shows "transport P a a (refl a) \ id (P`a)" + shows "transport P a a (refl a) \ id P`a" unfolding transport_def by derive declare @@ -423,13 +423,13 @@ schematic_goal transport_invl: "A: U i" "P: A \ U j" "x: A" "y: A" "p: x =[A] y" shows "?prf: - (transport[P, y, x] (inv[A, x, y] p)) o[P`x] (transport[P, x, y] p) =[P`x \ P`x] id(P`x)" + (transport[P, y, x] (inv[A, x, y] p)) o[P`x] (transport[P, x, y] p) =[P`x \ P`x] id P`x" proof (path_ind' x y p) fix x assume [intro]: "x: A" show - "refl (id (P`x)) : + "refl (id P`x) : transport[P, x, x] (inv[A, x, x] (refl x)) o[P`x] (transport[P, x, x] (refl x)) =[P`x \ P`x] - id (P`x)" + id P`x" by derive fix y p assume [intro]: "y: A" "p: x =[A] y" @@ -438,7 +438,7 @@ proof (path_ind' x y p) proof show "transport[P, x, y] p: P`x \ P`y" by routine qed routine show - "transport[P, y, x] (inv[A, x, y] p) o[P`x] transport[P, x, y] p =[P`x \ P`x] id (P`x): U j" + "transport[P, y, x] (inv[A, x, y] p) o[P`x] transport[P, x, y] p =[P`x \ P`x] id P`x: U j" by derive qed @@ -447,13 +447,13 @@ schematic_goal transport_invr: "A: U i" "P: A \ U j" "x: A" "y: A" "p: x =[A] y" shows "?prf: - (transport[P, x, y] p) o[P`y] (transport[P, y, x] (inv[A, x, y] p)) =[P`y \ P`y] id(P`y)" + (transport[P, x, y] p) o[P`y] (transport[P, y, x] (inv[A, x, y] p)) =[P`y \ P`y] id P`y" proof (path_ind' x y p) fix x assume [intro]: "x: A" show - "refl (id (P`x)) : + "refl (id P`x) : (transport[P, x, x] (refl x)) o[P`x] transport[P, x, x] (inv[A, x, x] (refl x)) =[P`x \ P`x] - id (P`x)" + id P`x" by derive fix y p assume [intro]: "y: A" "p: x =[A] y" @@ -462,7 +462,7 @@ proof (path_ind' x y p) proof show "transport[P, x, y] p: P`x \ P`y" by routine qed routine show - "transport[P, x, y] p o[P`y] transport[P, y, x] (inv[A, x, y] p) =[P`y \ P`y] id (P`y): U j" + "transport[P, x, y] p o[P`y] transport[P, y, x] (inv[A, x, y] p) =[P`y \ P`y] id P`y: U j" by derive qed -- cgit v1.2.3