From a1afde729f1d9b2f930696b117cfaec827eaa178 Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Wed, 12 Sep 2018 06:33:55 +0200 Subject: Some final touchups before release 0.1 for the MS thesis --- Coprod.thy | 2 +- EqualProps.thy | 4 ++-- ProdProps.thy | 2 +- Sum.thy | 2 +- Unit.thy | 2 +- Univalence.thy | 4 +++- 6 files changed, 9 insertions(+), 7 deletions(-) diff --git a/Coprod.thy b/Coprod.thy index b87958a..1ff7361 100644 --- a/Coprod.thy +++ b/Coprod.thy @@ -28,7 +28,7 @@ and \x. x: A \ c x: C (inl x); \y. y: B \ d y: C (inr y); u: A + B - \ \ ind\<^sub>+ c d u : C u" + \ \ ind\<^sub>+ c d u: C u" and Coprod_comp_inl: "\ C: A + B \ U i; diff --git a/EqualProps.thy b/EqualProps.thy index 4cfe280..5db8487 100644 --- a/EqualProps.thy +++ b/EqualProps.thy @@ -278,6 +278,8 @@ section \Transport\ definition transport :: "Term \ Term" where "transport p \ ind\<^sub>= (\x. (\<^bold>\x. x)) p" +text "Note that \transport\ is a polymorphic function in our formulation." + lemma transport_type: assumes "A: U i" "P: A \ U i" @@ -292,7 +294,5 @@ lemma transport_comp: shows "transport (refl x) \ id" unfolding transport_def by (derive lems: assms) -text "Note that in our formulation, \transport\ is a polymorphic function!" - end diff --git a/ProdProps.thy b/ProdProps.thy index 47e386b..a68f79b 100644 --- a/ProdProps.thy +++ b/ProdProps.thy @@ -14,7 +14,7 @@ begin section \Composition\ text " - The proof of associativity needs some guidance; it involves telling Isabelle to use the correct rule for \-type definitional equality, and the correct substitutions in the subgoals thereafter. + The proof of associativity needs some guidance; it involves telling Isabelle to use the correct rule for \-type definitional equality, and the correct substitutions in the subgoals thereafter. " lemma compose_assoc: diff --git a/Sum.thy b/Sum.thy index 6de20fd..aac81f7 100644 --- a/Sum.thy +++ b/Sum.thy @@ -47,7 +47,7 @@ and a: A; b: B a; \x y. \x: A; y: B(x)\ \ f x y: C ; - B: A \ U(i); + B: A \ U i; C: \x:A. B x \ U i \ \ ind\<^sub>\ f \ f a b" diff --git a/Unit.thy b/Unit.thy index 9b86739..6760f27 100644 --- a/Unit.thy +++ b/Unit.thy @@ -16,7 +16,7 @@ axiomatization pt :: Term ("\") and indUnit :: "[Term, Term] \ Term" ("(1ind\<^sub>\)") where - Unit_form: "\: U(O)" + Unit_form: "\: U O" and Unit_intro: "\: \" and diff --git a/Univalence.thy b/Univalence.thy index 80325f3..8599ba7 100644 --- a/Univalence.thy +++ b/Univalence.thy @@ -15,6 +15,8 @@ begin section \Homotopy and equivalence\ +text "We define polymorphic constants implementing the definitions of homotopy and equivalence." + axiomatization homotopic :: "[Term, Term] \ Term" (infix "~" 100) where homotopic_def: "\ f: \x:A. B x; @@ -166,7 +168,7 @@ proof qed -text "The univalence axiom:" +text "The univalence axiom." axiomatization univalence :: Term where ua: "univalence: isequiv idtoeqv" -- cgit v1.2.3