blob: 316841dafd61ae7e7a569163531e9d7543b2508b (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
|
(* Title: HoTT/HoTT_Methods.thy
Author: Josh Chen
Date: Jun 2018
Method setup for the HoTT library. Relies heavily on Eisbach.
*)
theory HoTT_Methods
imports
"HOL-Eisbach.Eisbach"
"HOL-Eisbach.Eisbach_Tools"
HoTT_Base
begin
section \<open>Method definitions\<close>
subsection \<open>Simple type rule proof search\<close>
text "
Prove type judgments \<open>A : U\<close> and inhabitation judgments \<open>a : A\<close> using the type rules declared [intro] and [elim] (in the respective theory files), as well as additional provided lemmas.
Can also perform typechecking, and search for elements of a type.
"
method simple uses lems = (assumption | rule lems | standard)+
subsection \<open>Wellformedness checker\<close>
text "
\<open>wellformed\<close> finds a proof of any valid typing judgment derivable from the judgments passed as \<open>lem\<close>.
The named theorem \<open>wellform\<close> is declared in HoTT_Base.thy.
"
method wellformed' uses jdmt declares wellform =
match wellform in rl: "PROP ?P" \<Rightarrow> \<open>(
catch \<open>rule rl[OF jdmt]\<close> \<open>fail\<close> |
catch \<open>wellformed' jdmt: rl[OF jdmt]\<close> \<open>fail\<close>
)\<close>
method wellformed uses lems =
match lems in lem: "?X : ?Y" \<Rightarrow> \<open>wellformed' jdmt: lem\<close>
subsection \<open>Derivation search\<close>
text " Combine \<open>simple\<close> and \<open>wellformed\<close> to search for derivations of judgments."
method derive uses lems = (simple lems: lems | wellformed lems: lems)+
subsection \<open>Substitution and simplification\<close>
text "Import the \<open>subst\<close> method, used for substituting definitional equalities."
ML_file "~~/src/Tools/misc_legacy.ML"
ML_file "~~/src/Tools/IsaPlanner/isand.ML"
ML_file "~~/src/Tools/IsaPlanner/rw_inst.ML"
ML_file "~~/src/Tools/IsaPlanner/zipper.ML"
ML_file "~~/src/Tools/eqsubst.ML"
text "Perform basic single-step computations:"
method compute uses lems = (subst lems comp)
end
|