aboutsummaryrefslogtreecommitdiff
path: root/Prod.thy
diff options
context:
space:
mode:
Diffstat (limited to 'Prod.thy')
-rw-r--r--Prod.thy4
1 files changed, 3 insertions, 1 deletions
diff --git a/Prod.thy b/Prod.thy
index 2cb62e4..aeddc49 100644
--- a/Prod.thy
+++ b/Prod.thy
@@ -117,7 +117,9 @@ lemma compose_assoc:
shows "(h o[B] g) o[A] f \<equiv> h o[A] g o[A] f"
unfolding compose_def by (derive lems: assms cong)
-abbreviation id :: "t \<Rightarrow> t" where "id A \<equiv> \<lambda>x: A. x"
+abbreviation id :: "t \<Rightarrow> t" ("(id _)" [115] 114) where "id A \<equiv> \<lambda>x: A. x"
+
+lemma id_type [intro]: "\<And>A. A: U i \<Longrightarrow> id A: A \<rightarrow> A" by derive
section \<open>Universal quantification\<close>