diff options
author | Josh Chen | 2018-07-03 18:57:57 +0200 |
---|---|---|
committer | Josh Chen | 2018-07-03 18:57:57 +0200 |
commit | 7823d59b2d9436f1bf0042fff62ee2bcc4c29ec0 (patch) | |
tree | e45df70f36abdedfa0e5c2bcaebfb11022b18a41 /ex | |
parent | 9ffa5ed2a972db4ae6274a7852de37945a32ab0e (diff) |
Refactor HoTT_Methods.thy, proved more stuff with new methods.
Diffstat (limited to 'ex')
-rw-r--r-- | ex/Methods.thy | 41 |
1 files changed, 41 insertions, 0 deletions
diff --git a/ex/Methods.thy b/ex/Methods.thy new file mode 100644 index 0000000..d174dde --- /dev/null +++ b/ex/Methods.thy @@ -0,0 +1,41 @@ +(* Title: HoTT/ex/Methods.thy + Author: Josh Chen + Date: Jul 2018 + +HoTT method usage examples +*) + +theory Methods + imports "../HoTT" +begin + +lemma + assumes "A : U" "B: A \<rightarrow> U" "\<And>x. x : A \<Longrightarrow> C x: B x \<rightarrow> U" + shows "\<Sum>x:A. \<Prod>y:B x. \<Sum>z:C x y. \<Prod>w:A. x =\<^sub>A w : U" +by (simple lems: assms) + + +lemma + assumes "f : \<Sum>x:A. \<Prod>y: B x. \<Sum>z: C x y. D x y z" + shows + "A : U" and + "B: A \<rightarrow> U" and + "\<And>x. x : A \<Longrightarrow> C x: B x \<rightarrow> U" and + "\<And>x y. \<lbrakk>x : A; y : B x\<rbrakk> \<Longrightarrow> D x y: C x y \<rightarrow> U" +proof - + show "A : U" by (wellformed jdgmt: assms) + show "B: A \<rightarrow> U" by (wellformed jdgmt: assms) + show "\<And>x. x : A \<Longrightarrow> C x: B x \<rightarrow> U" by (wellformed jdgmt: assms) + show "\<And>x y. \<lbrakk>x : A; y : B x\<rbrakk> \<Longrightarrow> D x y: C x y \<rightarrow> U" by (wellformed jdgmt: assms) +qed + + +text "Typechecking:" + +\<comment> \<open>Correctly determines the type of the pair\<close> +schematic_goal "\<lbrakk>a : A; b : B\<rbrakk> \<Longrightarrow> (a, b) : ?A" by simple + +\<comment> \<open>Finds element\<close> +schematic_goal "\<lbrakk>a : A; b : B\<rbrakk> \<Longrightarrow> ?x : A \<times> B" by simple + +end
\ No newline at end of file |