From b0ba102b783418560f9b7b15239681b11ea4c877 Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Tue, 26 May 2020 16:50:35 +0200 Subject: new material --- hott/Equivalence.thy | 15 ++++++++------- 1 file changed, 8 insertions(+), 7 deletions(-) (limited to 'hott/Equivalence.thy') diff --git a/hott/Equivalence.thy b/hott/Equivalence.thy index 2975738..9e7b83a 100644 --- a/hott/Equivalence.thy +++ b/hott/Equivalence.thy @@ -61,6 +61,8 @@ Lemma (derive) htrans: text \For calculations:\ +congruence "f ~ g" rhs g + lemmas homotopy_sym [sym] = hsym[rotated 4] and homotopy_trans [trans] = htrans[rotated 5] @@ -81,8 +83,8 @@ Lemma (derive) commute_homotopy: \ \Here it would really be nice to have automation for transport and propositional equality.\ apply (rule use_transport[where ?y="H x \ refl (g x)"]) - \ by (rule pathcomp_right_refl) - \ by (rule pathinv) (rule pathcomp_left_refl) + \ by (rule pathcomp_refl) + \ by (rule pathinv) (rule refl_pathcomp) \ by typechk done done @@ -256,12 +258,12 @@ Lemma (derive) biinv_imp_qinv: \ proof - have "g ~ g \ (id B)" by reduce refl - also have "g \ (id B) ~ g \ f \ h" + also have ".. ~ g \ f \ h" by (rule homotopy_funcomp_right) (rule \H2:_\[symmetric]) - also have "g \ f \ h ~ (id A) \ h" + also have ".. ~ (id A) \ h" by (subst funcomp_assoc[symmetric]) (rule homotopy_funcomp_left, rule \H1:_\) - also have "(id A) \ h ~ h" by reduce refl + also have ".. ~ h" by reduce refl finally have "g ~ h" by this then have "f \ g ~ f \ h" by (rule homotopy_funcomp_right) @@ -348,8 +350,7 @@ text \ \ Lemma - assumes - "A: U i" "B: U i" "p: A =\<^bsub>U i\<^esub> B" + assumes "A: U i" "B: U i" "p: A =\<^bsub>U i\<^esub> B" shows "A \ B" by (eq p) (rule equivalence_refl) -- cgit v1.2.3