aboutsummaryrefslogtreecommitdiff
path: root/HoTT_Base.thy
diff options
context:
space:
mode:
authorJosh Chen2018-06-27 16:10:07 +0200
committerJosh Chen2018-06-27 16:10:07 +0200
commit0d66c233b6dba82ffa93d7c060bcacc756284b25 (patch)
tree6f429ab15f13d360f8979b65c9343004efec215d /HoTT_Base.thy
parent4eca07fed1b54a59718dad04425527f9cc02af9f (diff)
Library organization and formatting
Diffstat (limited to '')
-rw-r--r--HoTT_Base.thy4
1 files changed, 3 insertions, 1 deletions
diff --git a/HoTT_Base.thy b/HoTT_Base.thy
index a0078fa..561dbe6 100644
--- a/HoTT_Base.thy
+++ b/HoTT_Base.thy
@@ -17,7 +17,7 @@ text "Set up type checking routines, proof methods etc."
section \<open>Metalogical definitions\<close>
text "A single meta-type \<open>Term\<close> suffices to implement the object-logic types and terms.
-We do not implement universes, and simply use \<open>a : U\<close> as a convenient shorthand to mean ``\<open>a\<close> is a type''."
+We do not implement universes, and simply use \<open>a : U\<close> as a convenient shorthand to mean ''\<open>a\<close> is a type''."
typedecl Term
@@ -32,6 +32,8 @@ consts
is_a_type :: "Term \<Rightarrow> prop" ("(1_ :/ U)" [0] 1000)
is_of_type :: "[Term, Term] \<Rightarrow> prop" ("(1_ :/ _)" [0, 0] 1000)
+text "The following fact is used to make explicit the assumption of well-formed contexts."
+
axiomatization where
inhabited_implies_type [intro, elim]: "\<And>a A. a : A \<Longrightarrow> A : U"