diff options
Diffstat (limited to 'HoTT_Base.thy')
-rw-r--r-- | HoTT_Base.thy | 3 |
1 files changed, 1 insertions, 2 deletions
diff --git a/HoTT_Base.thy b/HoTT_Base.thy index 7794601..a0078fa 100644 --- a/HoTT_Base.thy +++ b/HoTT_Base.thy @@ -7,7 +7,6 @@ Basic setup and definitions of a homotopy type theory object logic without unive theory HoTT_Base imports Pure - begin section \<open>Setup\<close> @@ -34,7 +33,7 @@ consts is_of_type :: "[Term, Term] \<Rightarrow> prop" ("(1_ :/ _)" [0, 0] 1000) axiomatization where - inhabited_implies_type [intro]: "\<And>a A. a : A \<Longrightarrow> A : U" + inhabited_implies_type [intro, elim]: "\<And>a A. a : A \<Longrightarrow> A : U" section \<open>Type families\<close> |