aboutsummaryrefslogtreecommitdiff
path: root/hott/More_Nat.thy
diff options
context:
space:
mode:
authorJosh Chen2020-07-21 02:16:14 +0200
committerGitHub2020-07-21 02:16:14 +0200
commitdfd241b2d85fc5a4ad4d7ddd64adf0138b05f083 (patch)
treeb4c4280b1bc4426059ddd184a2258d15d20a0bab /hott/More_Nat.thy
parent6aaf4d5b28a5284b3b02fa5c410d2d83a711840b (diff)
parent12eed8685674b7d5ff7bc45a44a061e01f99ce5f (diff)
Merge pull request #8 from jaycech3n/dev
Merge big diff on dev
Diffstat (limited to 'hott/More_Nat.thy')
-rw-r--r--hott/More_Nat.thy6
1 files changed, 3 insertions, 3 deletions
diff --git a/hott/More_Nat.thy b/hott/More_Nat.thy
index 8177170..59c8d54 100644
--- a/hott/More_Nat.thy
+++ b/hott/More_Nat.thy
@@ -15,15 +15,15 @@ Lemma (derive) eq: shows "Nat \<rightarrow> Nat \<rightarrow> U O"
apply intro focus vars n apply elim
\<guillemotright> by (rule TopF) \<comment> \<open>n \<equiv> 0\<close>
\<guillemotright> by (rule BotF) \<comment> \<open>n \<equiv> suc _\<close>
- \<guillemotright> by (rule U_in_U)
+ \<guillemotright> by (rule Ui_in_USi)
done
\<comment> \<open>m \<equiv> suc k\<close>
apply intro focus vars k k_eq n apply (elim n)
\<guillemotright> by (rule BotF) \<comment> \<open>n \<equiv> 0\<close>
\<guillemotright> prems vars l proof - show "k_eq l: U O" by typechk qed
- \<guillemotright> by (rule U_in_U)
+ \<guillemotright> by (rule Ui_in_USi)
done
- by (rule U_in_U)
+ by (rule Ui_in_USi)
done
text \<open>