aboutsummaryrefslogtreecommitdiff
path: root/EqualProps.thy
diff options
context:
space:
mode:
Diffstat (limited to 'EqualProps.thy')
-rw-r--r--EqualProps.thy4
1 files changed, 2 insertions, 2 deletions
diff --git a/EqualProps.thy b/EqualProps.thy
index 4cfe280..5db8487 100644
--- a/EqualProps.thy
+++ b/EqualProps.thy
@@ -278,6 +278,8 @@ section \<open>Transport\<close>
definition transport :: "Term \<Rightarrow> Term" where
"transport p \<equiv> ind\<^sub>= (\<lambda>x. (\<^bold>\<lambda>x. x)) p"
+text "Note that \<open>transport\<close> is a polymorphic function in our formulation."
+
lemma transport_type:
assumes
"A: U i" "P: A \<longrightarrow> U i"
@@ -292,7 +294,5 @@ lemma transport_comp:
shows "transport (refl x) \<equiv> id"
unfolding transport_def by (derive lems: assms)
-text "Note that in our formulation, \<open>transport\<close> is a polymorphic function!"
-
end