1975
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1 |
(*<*)
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
2 |
theory Paper
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
3 |
imports "Quotient"
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
4 |
"LaTeXsugar"
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
5 |
begin
|
1994
|
6 |
|
|
7 |
notation (latex output)
|
|
8 |
fun_rel ("_ ===> _" [51, 51] 50)
|
|
9 |
|
1975
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
10 |
(*>*)
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
11 |
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
12 |
section {* Introduction *}
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
13 |
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
14 |
text {* TBD *}
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
15 |
|
1978
|
16 |
subsection {* Contributions *}
|
1975
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
17 |
|
1978
|
18 |
text {*
|
|
19 |
We present the detailed lifting procedure, which was not shown before.
|
|
20 |
|
|
21 |
The quotient package presented in this paper has the following
|
|
22 |
advantages over existing packages:
|
|
23 |
\begin{itemize}
|
|
24 |
|
|
25 |
\item We define quotient composition, function map composition and
|
|
26 |
relation map composition. This lets lifting polymorphic types with
|
|
27 |
subtypes quotiented as well. We extend the notions of
|
|
28 |
respectfullness and preservation to cope with quotient
|
|
29 |
composition.
|
|
30 |
|
|
31 |
\item We allow lifting only some occurrences of quotiented
|
|
32 |
types. Rsp/Prs extended. (used in nominal)
|
|
33 |
|
|
34 |
\item We regularize more thanks to new lemmas. (inductions in
|
|
35 |
nominal).
|
|
36 |
|
|
37 |
\item The quotient package is very modular. Definitions can be added
|
|
38 |
separately, rsp and prs can be proved separately and theorems can
|
|
39 |
be lifted on a need basis. (useful with type-classes).
|
|
40 |
|
|
41 |
\item Can be used both manually (attribute, separate tactics,
|
|
42 |
rsp/prs databases) and programatically (automated definition of
|
|
43 |
lifted constants, the rsp proof obligations and theorem statement
|
|
44 |
translation according to given quotients).
|
|
45 |
|
|
46 |
\end{itemize}
|
|
47 |
*}
|
|
48 |
|
|
49 |
section {* Quotient Type*}
|
|
50 |
|
|
51 |
text {*
|
|
52 |
Defintion of quotient,
|
|
53 |
|
|
54 |
Equivalence,
|
|
55 |
|
|
56 |
Relation map and function map
|
|
57 |
*}
|
|
58 |
|
|
59 |
section {* Constants *}
|
|
60 |
|
|
61 |
text {*
|
|
62 |
Rep and Abs, Rsp and Prs
|
|
63 |
*}
|
|
64 |
|
|
65 |
section {* Lifting Theorems *}
|
|
66 |
|
1994
|
67 |
text {* TBD *}
|
|
68 |
|
|
69 |
text {* Why providing a statement to prove is necessary is some cases *}
|
|
70 |
|
|
71 |
subsection {* Regularization *}
|
|
72 |
|
|
73 |
text {*
|
|
74 |
Transformation of the theorem statement:
|
|
75 |
\begin{itemize}
|
|
76 |
\item Quantifiers and abstractions involving raw types replaced by bounded ones.
|
|
77 |
\item Equalities involving raw types replaced by bounded ones.
|
|
78 |
\end{itemize}
|
|
79 |
|
|
80 |
The procedure.
|
|
81 |
|
|
82 |
Example of non-regularizable theorem ($0 = 1$).
|
|
83 |
|
|
84 |
New regularization lemmas:
|
|
85 |
\begin{lemma}
|
|
86 |
If @{term R2} is an equivalence relation, then:
|
|
87 |
\begin{eqnarray}
|
|
88 |
@{thm (rhs) ball_reg_eqv_range[no_vars]} & = & @{thm (lhs) ball_reg_eqv_range[no_vars]}\\
|
|
89 |
@{thm (rhs) bex_reg_eqv_range[no_vars]} & = & @{thm (lhs) bex_reg_eqv_range[no_vars]}
|
|
90 |
\end{eqnarray}
|
|
91 |
\end{lemma}
|
|
92 |
|
|
93 |
*}
|
|
94 |
|
|
95 |
subsection {* Injection *}
|
|
96 |
|
|
97 |
subsection {* Cleaning *}
|
|
98 |
|
|
99 |
text {* Preservation of quantifiers, abstractions, relations, quotient-constants
|
|
100 |
(definitions) and user given constant preservation lemmas *}
|
|
101 |
|
|
102 |
section {* Examples *}
|
|
103 |
|
1978
|
104 |
section {* Related Work *}
|
|
105 |
|
|
106 |
text {*
|
|
107 |
\begin{itemize}
|
|
108 |
|
|
109 |
\item Peter Homeier's package (and related work from there), John
|
|
110 |
Harrison's one.
|
|
111 |
|
|
112 |
\item Manually defined quotients in Isabelle/HOL Library (Larry's
|
|
113 |
quotients, Markus's Quotient\_Type, Dixon's FSet, \ldots)
|
|
114 |
|
|
115 |
\item Oscar Slotosch defines quotient-type automatically but no
|
|
116 |
lifting.
|
|
117 |
|
|
118 |
\item PER. And how to avoid it.
|
|
119 |
|
|
120 |
\item Necessity of Hilbert Choice op.
|
|
121 |
|
|
122 |
\item Setoids in Coq
|
|
123 |
|
|
124 |
\end{itemize}
|
|
125 |
*}
|
1975
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
126 |
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
127 |
(*<*)
|
b1281a0051ae
added stub for quotient paper; call with isabelle make qpaper
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
128 |
end
|
1978
|
129 |
(*>*)
|