1 # |
1 # |
2 # IsaMakefile for HOL |
2 # approximative IsaMakefile for legacy applications |
3 # |
3 # |
4 |
|
5 ## targets |
|
6 |
4 |
7 default: HOL |
5 default: HOL |
8 |
6 |
9 images: \ |
7 clean: |
10 HOL \ |
8 -@$(ISABELLE_TOOL) build -a -n -c |
11 HOL-Library \ |
|
12 HOL-Algebra \ |
|
13 HOL-Boogie \ |
|
14 HOL-IMP \ |
|
15 HOL-Multivariate_Analysis \ |
|
16 HOL-NSA \ |
|
17 HOL-Nominal \ |
|
18 HOL-Proofs \ |
|
19 HOL-SPARK \ |
|
20 HOL-Word \ |
|
21 HOLCF \ |
|
22 IOA \ |
|
23 TLA \ |
|
24 HOL-Base \ |
|
25 HOL-Main \ |
|
26 HOL-Plain |
|
27 |
9 |
28 #Note: keep targets sorted |
10 all: |
29 test: \ |
11 @$(ISABELLE_TOOL) build -a |
30 HOL-Auth \ |
|
31 HOL-Bali \ |
|
32 HOL-Boogie-Examples \ |
|
33 HOL-Hahn_Banach \ |
|
34 HOL-Hoare \ |
|
35 HOL-Hoare_Parallel \ |
|
36 HOLCF-FOCUS \ |
|
37 HOLCF-IMP \ |
|
38 HOLCF-Library \ |
|
39 HOLCF-Tutorial \ |
|
40 HOLCF-ex \ |
|
41 HOL-IMPP \ |
|
42 HOL-Import \ |
|
43 HOL-IOA \ |
|
44 IOA-ABP \ |
|
45 IOA-NTP \ |
|
46 IOA-Storage \ |
|
47 IOA-ex \ |
|
48 HOL-Imperative_HOL \ |
|
49 HOL-Induct \ |
|
50 HOL-Isar_Examples \ |
|
51 HOL-Lattice \ |
|
52 HOL-Library-Codegenerator_Test \ |
|
53 HOL-Matrix_LP \ |
|
54 HOL-Metis_Examples \ |
|
55 HOL-MicroJava \ |
|
56 HOL-Mirabelle \ |
|
57 HOL-Mutabelle \ |
|
58 HOL-NanoJava \ |
|
59 HOL-Nitpick_Examples \ |
|
60 HOL-NSA-Examples \ |
|
61 HOL-Number_Theory \ |
|
62 HOL-Old_Number_Theory \ |
|
63 HOL-Quickcheck_Examples \ |
|
64 HOL-Quotient_Examples \ |
|
65 HOL-Predicate_Compile_Examples \ |
|
66 HOL-Prolog \ |
|
67 HOL-Proofs-ex \ |
|
68 HOL-Proofs-Lambda \ |
|
69 HOL-SET_Protocol \ |
|
70 HOL-SPARK-Examples \ |
|
71 HOL-SPARK-Manual \ |
|
72 HOL-Word-SMT_Examples \ |
|
73 HOL-Statespace \ |
|
74 TLA-Buffer \ |
|
75 TLA-Inc \ |
|
76 TLA-Memory \ |
|
77 HOL-TPTP \ |
|
78 HOL-UNITY \ |
|
79 HOL-Unix \ |
|
80 HOL-Word-Examples \ |
|
81 HOL-ZF |
|
82 # ^ this is the sort position |
|
83 |
|
84 benchmark: \ |
|
85 HOL-Datatype_Benchmark \ |
|
86 HOL-Quickcheck_Benchmark \ |
|
87 HOL-Record_Benchmark |
|
88 |
|
89 images-no-smlnj: \ |
|
90 HOL-Probability |
|
91 |
|
92 test-no-smlnj: \ |
|
93 HOL-ex \ |
|
94 HOL-Decision_Procs \ |
|
95 HOL-Proofs-Extraction \ |
|
96 HOL-Nominal-Examples |
|
97 |
|
98 all: test-no-smlnj test images-no-smlnj images |
|
99 full: all benchmark |
|
100 smlnj: test images |
|
101 |
|
102 |
|
103 ## global settings |
|
104 |
|
105 SRC = $(ISABELLE_HOME)/src |
|
106 OUT = $(ISABELLE_OUTPUT) |
|
107 LOG = $(OUT)/log |
|
108 |
|
109 |
|
110 ## HOL |
|
111 |
|
112 HOL: Pure $(OUT)/HOL |
|
113 |
|
114 HOL-Base: Pure $(OUT)/HOL-Base |
|
115 |
|
116 HOL-Plain: Pure $(OUT)/HOL-Plain |
|
117 |
|
118 HOL-Main: Pure $(OUT)/HOL-Main |
|
119 |
12 |
120 Pure: |
13 Pure: |
121 @cd $(SRC)/Pure; $(ISABELLE_TOOL) make Pure |
14 @$(ISABELLE_TOOL) build -b Pure |
122 |
15 |
123 $(OUT)/Pure: Pure |
16 HOL: |
|
17 @$(ISABELLE_TOOL) build -b HOL |
124 |
18 |
125 BASE_DEPENDENCIES = $(OUT)/Pure \ |
19 HOL-Library: |
126 $(SRC)/Provers/blast.ML \ |
20 @$(ISABELLE_TOOL) build -b HOL-Library |
127 $(SRC)/Provers/clasimp.ML \ |
|
128 $(SRC)/Provers/classical.ML \ |
|
129 $(SRC)/Provers/hypsubst.ML \ |
|
130 $(SRC)/Provers/quantifier1.ML \ |
|
131 $(SRC)/Provers/splitter.ML \ |
|
132 $(SRC)/Tools/Code/code_haskell.ML \ |
|
133 $(SRC)/Tools/Code/code_ml.ML \ |
|
134 $(SRC)/Tools/Code/code_namespace.ML \ |
|
135 $(SRC)/Tools/Code/code_preproc.ML \ |
|
136 $(SRC)/Tools/Code/code_printer.ML \ |
|
137 $(SRC)/Tools/Code/code_runtime.ML \ |
|
138 $(SRC)/Tools/Code/code_scala.ML \ |
|
139 $(SRC)/Tools/Code/code_simp.ML \ |
|
140 $(SRC)/Tools/Code/code_target.ML \ |
|
141 $(SRC)/Tools/Code/code_thingol.ML \ |
|
142 $(SRC)/Tools/Code_Generator.thy \ |
|
143 $(SRC)/Tools/IsaPlanner/isand.ML \ |
|
144 $(SRC)/Tools/IsaPlanner/rw_inst.ML \ |
|
145 $(SRC)/Tools/IsaPlanner/rw_tools.ML \ |
|
146 $(SRC)/Tools/IsaPlanner/zipper.ML \ |
|
147 $(SRC)/Tools/atomize_elim.ML \ |
|
148 $(SRC)/Tools/cache_io.ML \ |
|
149 $(SRC)/Tools/case_product.ML \ |
|
150 $(SRC)/Tools/coherent.ML \ |
|
151 $(SRC)/Tools/cong_tac.ML \ |
|
152 $(SRC)/Tools/eqsubst.ML \ |
|
153 $(SRC)/Tools/induct.ML \ |
|
154 $(SRC)/Tools/induct_tacs.ML \ |
|
155 $(SRC)/Tools/induction.ML \ |
|
156 $(SRC)/Tools/intuitionistic.ML \ |
|
157 $(SRC)/Tools/misc_legacy.ML \ |
|
158 $(SRC)/Tools/nbe.ML \ |
|
159 $(SRC)/Tools/project_rule.ML \ |
|
160 $(SRC)/Tools/quickcheck.ML \ |
|
161 $(SRC)/Tools/solve_direct.ML \ |
|
162 $(SRC)/Tools/subtyping.ML \ |
|
163 $(SRC)/Tools/try.ML \ |
|
164 $(SRC)/Tools/value.ML \ |
|
165 HOL.thy \ |
|
166 Tools/hologic.ML \ |
|
167 Tools/simpdata.ML |
|
168 |
21 |
169 $(OUT)/HOL-Base: base.ML $(BASE_DEPENDENCIES) |
22 HOL-IMP: |
170 @$(ISABELLE_TOOL) usedir -b -f base.ML -d false -g false $(OUT)/Pure HOL-Base |
23 @$(ISABELLE_TOOL) build -b HOL-IMP |
171 |
24 |
172 PLAIN_DEPENDENCIES = $(BASE_DEPENDENCIES) \ |
25 HOL-Multivariate_Analysis: |
173 $(SRC)/Provers/Arith/cancel_div_mod.ML \ |
26 @$(ISABELLE_TOOL) build -b HOL-Multivariate_Analysis |
174 $(SRC)/Provers/Arith/fast_lin_arith.ML \ |
|
175 $(SRC)/Provers/order.ML \ |
|
176 $(SRC)/Provers/trancl.ML \ |
|
177 $(SRC)/Tools/Metis/metis.ML \ |
|
178 $(SRC)/Tools/rat.ML \ |
|
179 ATP.thy \ |
|
180 Complete_Lattices.thy \ |
|
181 Complete_Partial_Order.thy \ |
|
182 Datatype.thy \ |
|
183 Extraction.thy \ |
|
184 Fields.thy \ |
|
185 Finite_Set.thy \ |
|
186 Fun.thy \ |
|
187 FunDef.thy \ |
|
188 Groups.thy \ |
|
189 Inductive.thy \ |
|
190 Lattices.thy \ |
|
191 Meson.thy \ |
|
192 Metis.thy \ |
|
193 Nat.thy \ |
|
194 Num.thy \ |
|
195 Option.thy \ |
|
196 Orderings.thy \ |
|
197 Partial_Function.thy \ |
|
198 Plain.thy \ |
|
199 Power.thy \ |
|
200 Product_Type.thy \ |
|
201 Relation.thy \ |
|
202 Rings.thy \ |
|
203 SAT.thy \ |
|
204 Set.thy \ |
|
205 Sum_Type.thy \ |
|
206 Tools/ATP/atp_problem.ML \ |
|
207 Tools/ATP/atp_problem_generate.ML \ |
|
208 Tools/ATP/atp_proof.ML \ |
|
209 Tools/ATP/atp_proof_reconstruct.ML \ |
|
210 Tools/ATP/atp_proof_redirect.ML \ |
|
211 Tools/ATP/atp_systems.ML \ |
|
212 Tools/ATP/atp_util.ML \ |
|
213 Tools/Datatype/datatype.ML \ |
|
214 Tools/Datatype/datatype_aux.ML \ |
|
215 Tools/Datatype/datatype_case.ML \ |
|
216 Tools/Datatype/datatype_codegen.ML \ |
|
217 Tools/Datatype/datatype_data.ML \ |
|
218 Tools/Datatype/datatype_prop.ML \ |
|
219 Tools/Datatype/datatype_realizer.ML \ |
|
220 Tools/Datatype/primrec.ML \ |
|
221 Tools/Datatype/rep_datatype.ML \ |
|
222 Tools/Function/context_tree.ML \ |
|
223 Tools/Function/fun.ML \ |
|
224 Tools/Function/function.ML \ |
|
225 Tools/Function/function_common.ML \ |
|
226 Tools/Function/function_core.ML \ |
|
227 Tools/Function/function_lib.ML \ |
|
228 Tools/Function/induction_schema.ML \ |
|
229 Tools/Function/lexicographic_order.ML \ |
|
230 Tools/Function/measure_functions.ML \ |
|
231 Tools/Function/mutual.ML \ |
|
232 Tools/Function/partial_function.ML \ |
|
233 Tools/Function/pat_completeness.ML \ |
|
234 Tools/Function/pattern_split.ML \ |
|
235 Tools/Function/relation.ML \ |
|
236 Tools/Function/scnp_reconstruct.ML \ |
|
237 Tools/Function/scnp_solve.ML \ |
|
238 Tools/Function/size.ML \ |
|
239 Tools/Function/sum_tree.ML \ |
|
240 Tools/Function/termination.ML \ |
|
241 Tools/Meson/meson.ML \ |
|
242 Tools/Meson/meson_clausify.ML \ |
|
243 Tools/Meson/meson_tactic.ML \ |
|
244 Tools/Metis/metis_generate.ML \ |
|
245 Tools/Metis/metis_reconstruct.ML \ |
|
246 Tools/Metis/metis_tactic.ML \ |
|
247 Tools/arith_data.ML \ |
|
248 Tools/cnf_funcs.ML \ |
|
249 Tools/enriched_type.ML \ |
|
250 Tools/group_cancel.ML \ |
|
251 Tools/inductive.ML \ |
|
252 Tools/inductive_realizer.ML \ |
|
253 Tools/inductive_set.ML \ |
|
254 Tools/lambda_lifting.ML \ |
|
255 Tools/lin_arith.ML \ |
|
256 Tools/monomorph.ML \ |
|
257 Tools/nat_arith.ML \ |
|
258 Tools/prop_logic.ML \ |
|
259 Tools/refute.ML \ |
|
260 Tools/rewrite_hol_proof.ML \ |
|
261 Tools/sat_funcs.ML \ |
|
262 Tools/sat_solver.ML \ |
|
263 Tools/set_comprehension_pointfree.ML \ |
|
264 Tools/split_rule.ML \ |
|
265 Tools/try0.ML \ |
|
266 Tools/typedef.ML \ |
|
267 Transitive_Closure.thy \ |
|
268 Typedef.thy \ |
|
269 Wellfounded.thy |
|
270 |
27 |
271 $(OUT)/HOL-Plain: plain.ML $(PLAIN_DEPENDENCIES) |
28 HOL-Nominal: |
272 @$(ISABELLE_TOOL) usedir -b -f plain.ML -g true $(OUT)/Pure HOL-Plain |
29 @$(ISABELLE_TOOL) build -b HOL-Nominal |
273 |
30 |
274 MAIN_DEPENDENCIES = $(PLAIN_DEPENDENCIES) \ |
31 HOL-Word: |
275 Big_Operators.thy \ |
32 @$(ISABELLE_TOOL) build -b HOL-Word |
276 Code_Evaluation.thy \ |
|
277 Code_Numeral.thy \ |
|
278 Divides.thy \ |
|
279 DSequence.thy \ |
|
280 Equiv_Relations.thy \ |
|
281 Enum.thy \ |
|
282 Groebner_Basis.thy \ |
|
283 Hilbert_Choice.thy \ |
|
284 Int.thy \ |
|
285 Lazy_Sequence.thy \ |
|
286 Lifting.thy \ |
|
287 List.thy \ |
|
288 Main.thy \ |
|
289 Map.thy \ |
|
290 Nat_Transfer.thy \ |
|
291 New_DSequence.thy \ |
|
292 New_Random_Sequence.thy \ |
|
293 Nitpick.thy \ |
|
294 Numeral_Simprocs.thy \ |
|
295 Presburger.thy \ |
|
296 Predicate.thy \ |
|
297 Predicate_Compile.thy \ |
|
298 Quickcheck.thy \ |
|
299 Quickcheck_Exhaustive.thy \ |
|
300 Quickcheck_Narrowing.thy \ |
|
301 Quotient.thy \ |
|
302 Random.thy \ |
|
303 Random_Sequence.thy \ |
|
304 Record.thy \ |
|
305 Refute.thy \ |
|
306 Semiring_Normalization.thy \ |
|
307 Set_Interval.thy \ |
|
308 Sledgehammer.thy \ |
|
309 SMT.thy \ |
|
310 String.thy \ |
|
311 Transfer.thy \ |
|
312 Typerep.thy \ |
|
313 $(SRC)/Provers/Arith/assoc_fold.ML \ |
|
314 $(SRC)/Provers/Arith/cancel_numeral_factor.ML \ |
|
315 $(SRC)/Provers/Arith/cancel_numerals.ML \ |
|
316 $(SRC)/Provers/Arith/combine_numerals.ML \ |
|
317 $(SRC)/Provers/Arith/extract_common_term.ML \ |
|
318 Tools/choice_specification.ML \ |
|
319 Tools/code_evaluation.ML \ |
|
320 Tools/groebner.ML \ |
|
321 Tools/int_arith.ML \ |
|
322 Tools/legacy_transfer.ML \ |
|
323 Tools/Lifting/lifting_def.ML \ |
|
324 Tools/Lifting/lifting_info.ML \ |
|
325 Tools/Lifting/lifting_term.ML \ |
|
326 Tools/Lifting/lifting_setup.ML \ |
|
327 Tools/list_code.ML \ |
|
328 Tools/list_to_set_comprehension.ML \ |
|
329 Tools/nat_numeral_simprocs.ML \ |
|
330 Tools/Nitpick/kodkod.ML \ |
|
331 Tools/Nitpick/kodkod_sat.ML \ |
|
332 Tools/Nitpick/nitpick.ML \ |
|
333 Tools/Nitpick/nitpick_hol.ML \ |
|
334 Tools/Nitpick/nitpick_isar.ML \ |
|
335 Tools/Nitpick/nitpick_kodkod.ML \ |
|
336 Tools/Nitpick/nitpick_model.ML \ |
|
337 Tools/Nitpick/nitpick_mono.ML \ |
|
338 Tools/Nitpick/nitpick_nut.ML \ |
|
339 Tools/Nitpick/nitpick_peephole.ML \ |
|
340 Tools/Nitpick/nitpick_preproc.ML \ |
|
341 Tools/Nitpick/nitpick_rep.ML \ |
|
342 Tools/Nitpick/nitpick_scope.ML \ |
|
343 Tools/Nitpick/nitpick_tests.ML \ |
|
344 Tools/Nitpick/nitpick_util.ML \ |
|
345 Tools/numeral.ML \ |
|
346 Tools/numeral_simprocs.ML \ |
|
347 Tools/Predicate_Compile/core_data.ML \ |
|
348 Tools/Predicate_Compile/mode_inference.ML \ |
|
349 Tools/Predicate_Compile/predicate_compile_aux.ML \ |
|
350 Tools/Predicate_Compile/predicate_compile_compilations.ML \ |
|
351 Tools/Predicate_Compile/predicate_compile_core.ML \ |
|
352 Tools/Predicate_Compile/predicate_compile_data.ML \ |
|
353 Tools/Predicate_Compile/predicate_compile_fun.ML \ |
|
354 Tools/Predicate_Compile/predicate_compile.ML \ |
|
355 Tools/Predicate_Compile/predicate_compile_proof.ML \ |
|
356 Tools/Predicate_Compile/predicate_compile_specialisation.ML \ |
|
357 Tools/Predicate_Compile/predicate_compile_pred.ML \ |
|
358 Tools/Qelim/cooper.ML \ |
|
359 Tools/Qelim/cooper_procedure.ML \ |
|
360 Tools/Qelim/qelim.ML \ |
|
361 Tools/Quickcheck/exhaustive_generators.ML \ |
|
362 Tools/Quickcheck/random_generators.ML \ |
|
363 Tools/Quickcheck/quickcheck_common.ML \ |
|
364 Tools/Quickcheck/narrowing_generators.ML \ |
|
365 Tools/Quickcheck/Narrowing_Engine.hs \ |
|
366 Tools/Quickcheck/PNF_Narrowing_Engine.hs \ |
|
367 Tools/Quotient/quotient_def.ML \ |
|
368 Tools/Quotient/quotient_info.ML \ |
|
369 Tools/Quotient/quotient_tacs.ML \ |
|
370 Tools/Quotient/quotient_term.ML \ |
|
371 Tools/Quotient/quotient_type.ML \ |
|
372 Tools/record.ML \ |
|
373 Tools/semiring_normalizer.ML \ |
|
374 Tools/Sledgehammer/async_manager.ML \ |
|
375 Tools/Sledgehammer/sledgehammer_fact.ML \ |
|
376 Tools/Sledgehammer/sledgehammer_mash.ML \ |
|
377 Tools/Sledgehammer/sledgehammer_mepo.ML \ |
|
378 Tools/Sledgehammer/sledgehammer_minimize.ML \ |
|
379 Tools/Sledgehammer/sledgehammer_isar.ML \ |
|
380 Tools/Sledgehammer/sledgehammer_provers.ML \ |
|
381 Tools/Sledgehammer/sledgehammer_run.ML \ |
|
382 Tools/Sledgehammer/sledgehammer_util.ML \ |
|
383 Tools/SMT/smtlib_interface.ML \ |
|
384 Tools/SMT/smt_builtin.ML \ |
|
385 Tools/SMT/smt_config.ML \ |
|
386 Tools/SMT/smt_datatypes.ML \ |
|
387 Tools/SMT/smt_failure.ML \ |
|
388 Tools/SMT/smt_normalize.ML \ |
|
389 Tools/SMT/smt_setup_solvers.ML \ |
|
390 Tools/SMT/smt_solver.ML \ |
|
391 Tools/SMT/smt_translate.ML \ |
|
392 Tools/SMT/smt_utils.ML \ |
|
393 Tools/SMT/z3_interface.ML \ |
|
394 Tools/SMT/z3_model.ML \ |
|
395 Tools/SMT/z3_proof_literals.ML \ |
|
396 Tools/SMT/z3_proof_methods.ML \ |
|
397 Tools/SMT/z3_proof_parser.ML \ |
|
398 Tools/SMT/z3_proof_reconstruction.ML \ |
|
399 Tools/SMT/z3_proof_tools.ML \ |
|
400 Tools/string_code.ML \ |
|
401 Tools/string_syntax.ML \ |
|
402 Tools/transfer.ML \ |
|
403 |
33 |
404 $(OUT)/HOL-Main: main.ML $(MAIN_DEPENDENCIES) |
34 HOLCF: |
405 @$(ISABELLE_TOOL) usedir -b -f main.ML -g true $(OUT)/Pure HOL-Main |
35 @$(ISABELLE_TOOL) build -b HOLCF |
406 |
36 |
407 HOL_DEPENDENCIES = $(MAIN_DEPENDENCIES) \ |
|
408 Archimedean_Field.thy \ |
|
409 Complex.thy \ |
|
410 Complex_Main.thy \ |
|
411 Deriv.thy \ |
|
412 Fact.thy \ |
|
413 GCD.thy \ |
|
414 Lim.thy \ |
|
415 Limits.thy \ |
|
416 Ln.thy \ |
|
417 Log.thy \ |
|
418 Lubs.thy \ |
|
419 MacLaurin.thy \ |
|
420 NthRoot.thy \ |
|
421 Parity.thy \ |
|
422 RComplete.thy \ |
|
423 Rat.thy \ |
|
424 Real.thy \ |
|
425 RealDef.thy \ |
|
426 RealVector.thy \ |
|
427 SEQ.thy \ |
|
428 Series.thy \ |
|
429 SupInf.thy \ |
|
430 Taylor.thy \ |
|
431 Tools/SMT/smt_real.ML \ |
|
432 Tools/float_syntax.ML \ |
|
433 Transcendental.thy |
|
434 |
|
435 $(OUT)/HOL: ROOT.ML $(HOL_DEPENDENCIES) |
|
436 @$(ISABELLE_TOOL) usedir -b -g true $(OUT)/Pure HOL |
|
437 |
|
438 |
|
439 ## HOL-Library |
|
440 |
|
441 HOL-Library: HOL $(OUT)/HOL-Library |
|
442 |
|
443 $(OUT)/HOL-Library: $(OUT)/HOL Library/ROOT.ML \ |
|
444 $(SRC)/HOL/Tools/float_arith.ML $(SRC)/Tools/float.ML \ |
|
445 Library/Abstract_Rat.thy $(SRC)/Tools/Adhoc_Overloading.thy \ |
|
446 Library/AList.thy Library/AList_Mapping.thy \ |
|
447 Library/BigO.thy Library/Binomial.thy \ |
|
448 Library/Bit.thy Library/Boolean_Algebra.thy Library/Cardinality.thy \ |
|
449 Library/Char_nat.thy Library/Code_Char.thy Library/Code_Char_chr.thy \ |
|
450 Library/Code_Char_ord.thy Library/Code_Integer.thy \ |
|
451 Library/Code_Nat.thy Library/Code_Natural.thy \ |
|
452 Library/Efficient_Nat.thy Library/Code_Prolog.thy \ |
|
453 Library/Code_Real_Approx_By_Float.thy \ |
|
454 Tools/Predicate_Compile/code_prolog.ML Library/ContNotDenum.thy \ |
|
455 Library/Continuity.thy \ |
|
456 Library/Convex.thy Library/Countable.thy \ |
|
457 Library/Debug.thy \ |
|
458 Library/Dlist.thy Library/Eval_Witness.thy \ |
|
459 Library/DAList.thy Library/Dlist.thy \ |
|
460 Library/Eval_Witness.thy \ |
|
461 Library/Extended_Real.thy Library/Extended_Nat.thy \ |
|
462 Library/FinFun.thy Library/FinFun_Syntax.thy Library/Float.thy \ |
|
463 Library/Formal_Power_Series.thy Library/Fraction_Field.thy \ |
|
464 Library/FrechetDeriv.thy Library/FuncSet.thy \ |
|
465 Library/Function_Algebras.thy Library/Function_Division.thy \ |
|
466 Library/Fundamental_Theorem_Algebra.thy \ |
|
467 Library/Glbs.thy Library/Indicator_Function.thy \ |
|
468 Library/Infinite_Set.thy Library/Inner_Product.thy \ |
|
469 Library/Kleene_Algebra.thy Library/LaTeXsugar.thy \ |
|
470 Library/Lattice_Algebras.thy Library/Lattice_Syntax.thy \ |
|
471 Library/Library.thy Library/List_Prefix.thy \ |
|
472 Library/List_lexord.thy Library/Mapping.thy Library/Monad_Syntax.thy \ |
|
473 Library/Multiset.thy Library/Nat_Bijection.thy \ |
|
474 Library/Numeral_Type.thy Library/Old_Recdef.thy \ |
|
475 Library/OptionalSugar.thy Library/Order_Relation.thy \ |
|
476 Library/Parallel.thy \ |
|
477 Library/Permutation.thy Library/Permutations.thy \ |
|
478 Library/Phantom_Type.thy Library/Poly_Deriv.thy \ |
|
479 Library/Polynomial.thy Library/Predicate_Compile_Quickcheck.thy \ |
|
480 Library/Preorder.thy Library/Product_Vector.thy \ |
|
481 Library/Product_ord.thy Library/Product_plus.thy \ |
|
482 Library/Product_Lattice.thy Library/Quickcheck_Types.thy \ |
|
483 Library/Quotient_List.thy Library/Quotient_Option.thy \ |
|
484 Library/Quotient_Product.thy Library/Quotient_Set.thy \ |
|
485 Library/Quotient_Sum.thy Library/Quotient_Syntax.thy \ |
|
486 Library/Quotient_Type.thy Library/RBT.thy Library/RBT_Impl.thy \ |
|
487 Library/RBT_Mapping.thy Library/README.html Library/Saturated.thy \ |
|
488 Library/Set_Algebras.thy Library/State_Monad.thy Library/Ramsey.thy \ |
|
489 Library/Reflection.thy Library/Sublist_Order.thy \ |
|
490 Library/Sum_of_Squares.thy Library/Sum_of_Squares/sos_wrapper.ML \ |
|
491 Library/Sum_of_Squares/sum_of_squares.ML Library/Target_Numeral.thy \ |
|
492 Library/Transitive_Closure_Table.thy Library/Univ_Poly.thy \ |
|
493 Library/Wfrec.thy Library/While_Combinator.thy Library/Zorn.thy \ |
|
494 $(SRC)/Tools/adhoc_overloading.ML Library/positivstellensatz.ML \ |
|
495 Library/reflection.ML Library/reify_data.ML \ |
|
496 Library/document/root.bib Library/document/root.tex \ |
|
497 Tools/TFL/casesplit.ML Tools/TFL/dcterm.ML Tools/TFL/post.ML \ |
|
498 Tools/TFL/rules.ML Tools/TFL/tfl.ML Tools/TFL/thms.ML \ |
|
499 Tools/TFL/thry.ML Tools/TFL/usyntax.ML Tools/TFL/utils.ML \ |
|
500 Tools/recdef.ML |
|
501 @cd Library; $(ISABELLE_TOOL) usedir -b $(OUT)/HOL HOL-Library |
|
502 |
|
503 |
|
504 ## HOL-Hahn_Banach |
|
505 |
|
506 HOL-Hahn_Banach: HOL $(LOG)/HOL-Hahn_Banach.gz |
|
507 |
|
508 $(LOG)/HOL-Hahn_Banach.gz: $(OUT)/HOL Hahn_Banach/Bounds.thy \ |
|
509 Hahn_Banach/Function_Norm.thy Hahn_Banach/Function_Order.thy \ |
|
510 Hahn_Banach/Hahn_Banach.thy Hahn_Banach/Hahn_Banach_Ext_Lemmas.thy \ |
|
511 Hahn_Banach/Hahn_Banach_Sup_Lemmas.thy Hahn_Banach/Linearform.thy \ |
|
512 Hahn_Banach/Normed_Space.thy Hahn_Banach/README.html \ |
|
513 Hahn_Banach/ROOT.ML Hahn_Banach/Subspace.thy \ |
|
514 Hahn_Banach/Vector_Space.thy Hahn_Banach/Zorn_Lemma.thy \ |
|
515 Hahn_Banach/document/root.bib Hahn_Banach/document/root.tex |
|
516 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Hahn_Banach |
|
517 |
|
518 |
|
519 ## HOL-Induct |
|
520 |
|
521 HOL-Induct: HOL $(LOG)/HOL-Induct.gz |
|
522 |
|
523 $(LOG)/HOL-Induct.gz: $(OUT)/HOL Induct/Com.thy Induct/Comb.thy \ |
|
524 Induct/Ordinals.thy Induct/PropLog.thy Induct/QuoNestedDataType.thy \ |
|
525 Induct/QuoDataType.thy Induct/ROOT.ML Induct/Sexp.thy \ |
|
526 Induct/Sigma_Algebra.thy Induct/ABexp.thy Induct/SList.thy \ |
|
527 Induct/Term.thy Induct/Tree.thy Induct/document/root.tex |
|
528 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Induct |
|
529 |
|
530 |
|
531 ## HOL-IMP |
|
532 |
|
533 HOL-IMP: HOL $(OUT)/HOL-IMP |
|
534 |
|
535 $(OUT)/HOL-IMP: $(OUT)/HOL \ |
|
536 IMP/ACom.thy \ |
|
537 IMP/Abs_Int0.thy IMP/Abs_State.thy IMP/Abs_Int1.thy \ |
|
538 IMP/Abs_Int1_const.thy IMP/Abs_Int1_parity.thy \ |
|
539 IMP/Abs_Int2.thy IMP/Abs_Int2_ivl.thy IMP/Abs_Int3.thy \ |
|
540 IMP/Abs_Int_ITP/Abs_Int0_ITP.thy IMP/Abs_Int_ITP/Abs_State_ITP.thy \ |
|
541 IMP/Abs_Int_ITP/Abs_Int1_ITP.thy IMP/Abs_Int_ITP/Abs_Int1_const_ITP.thy \ |
|
542 IMP/Abs_Int_ITP/Abs_Int1_parity_ITP.thy IMP/Abs_Int_ITP/Abs_Int2_ITP.thy \ |
|
543 IMP/Abs_Int_ITP/Abs_Int2_ivl_ITP.thy IMP/Abs_Int_ITP/Abs_Int3_ITP.thy \ |
|
544 IMP/Abs_Int_Den/Abs_Int_den0_fun.thy \ |
|
545 IMP/Abs_Int_Den/Abs_State_den.thy IMP/Abs_Int_Den/Abs_Int_den0.thy \ |
|
546 IMP/Abs_Int_Den/Abs_Int_den0_const.thy IMP/Abs_Int_Den/Abs_Int_den1.thy \ |
|
547 IMP/Abs_Int_Den/Abs_Int_den1_ivl.thy IMP/Abs_Int_Den/Abs_Int_den2.thy \ |
|
548 IMP/ASM.thy IMP/AExp.thy IMP/BExp.thy IMP/Big_Step.thy IMP/C_like.thy \ |
|
549 IMP/Collecting.thy IMP/Collecting_list.thy IMP/Collecting1.thy IMP/Com.thy \ |
|
550 IMP/Compiler.thy IMP/Comp_Rev.thy \ |
|
551 IMP/Def_Ass.thy IMP/Def_Ass_Big.thy IMP/Def_Ass_Exp.thy \ |
|
552 IMP/Def_Ass_Small.thy IMP/Def_Ass_Sound_Big.thy \ |
|
553 IMP/Def_Ass_Sound_Small.thy IMP/Denotation.thy IMP/Hoare.thy \ |
|
554 IMP/HoareT.thy IMP/Hoare_Examples.thy IMP/Hoare_Sound_Complete.thy \ |
|
555 IMP/Live.thy IMP/Live_True.thy IMP/OO.thy IMP/Poly_Types.thy IMP/Procs.thy \ |
|
556 IMP/Procs_Dyn_Vars_Dyn.thy IMP/Procs_Stat_Vars_Dyn.thy \ |
|
557 IMP/Procs_Stat_Vars_Stat.thy IMP/Sec_Type_Expr.thy IMP/Sec_Typing.thy \ |
|
558 IMP/Sec_TypingT.thy IMP/Small_Step.thy IMP/Star.thy IMP/Types.thy \ |
|
559 IMP/VC.thy IMP/Vars.thy \ |
|
560 IMP/ROOT.ML IMP/document/root.tex IMP/document/root.bib |
|
561 @cd IMP && $(ISABELLE_TOOL) usedir -g true -b $(OUT)/HOL HOL-IMP |
|
562 |
|
563 ## HOL-IMPP |
|
564 |
|
565 HOL-IMPP: HOL $(LOG)/HOL-IMPP.gz |
|
566 |
|
567 $(LOG)/HOL-IMPP.gz: $(OUT)/HOL IMPP/ROOT.ML IMPP/Com.thy \ |
|
568 IMPP/Natural.thy IMPP/Hoare.thy IMPP/Misc.thy IMPP/EvenOdd.thy |
|
569 @$(ISABELLE_TOOL) usedir $(OUT)/HOL IMPP |
|
570 |
|
571 |
|
572 ## HOL-Import |
|
573 |
|
574 HOL-Import: $(LOG)/HOL-Import.gz |
|
575 |
|
576 $(LOG)/HOL-Import.gz: $(OUT)/HOL \ |
|
577 Import/ROOT.ML \ |
|
578 Import/Import_Setup.thy \ |
|
579 Import/import_data.ML \ |
|
580 Import/import_rule.ML \ |
|
581 Import/HOL_Light_Maps.thy \ |
|
582 Import/HOL_Light_Import.thy |
|
583 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Import |
|
584 |
|
585 |
|
586 ## HOL-Number_Theory |
|
587 |
|
588 HOL-Number_Theory: HOL $(LOG)/HOL-Number_Theory.gz |
|
589 |
|
590 $(LOG)/HOL-Number_Theory.gz: $(OUT)/HOL $(ALGEBRA_DEPENDENCIES) \ |
|
591 Library/Multiset.thy \ |
|
592 Number_Theory/Binomial.thy \ |
|
593 Number_Theory/Cong.thy \ |
|
594 Number_Theory/Fib.thy \ |
|
595 Number_Theory/MiscAlgebra.thy \ |
|
596 Number_Theory/Number_Theory.thy \ |
|
597 Number_Theory/Residues.thy \ |
|
598 Number_Theory/UniqueFactorization.thy \ |
|
599 Number_Theory/ROOT.ML |
|
600 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Number_Theory |
|
601 |
|
602 |
|
603 ## HOL-Old_Number_Theory |
|
604 |
|
605 HOL-Old_Number_Theory: HOL $(LOG)/HOL-Old_Number_Theory.gz |
|
606 |
|
607 $(LOG)/HOL-Old_Number_Theory.gz: $(OUT)/HOL Library/Permutation.thy \ |
|
608 Old_Number_Theory/Primes.thy Old_Number_Theory/Fib.thy \ |
|
609 Old_Number_Theory/Factorization.thy Old_Number_Theory/BijectionRel.thy\ |
|
610 Old_Number_Theory/Chinese.thy Old_Number_Theory/EulerFermat.thy \ |
|
611 Old_Number_Theory/IntFact.thy Old_Number_Theory/IntPrimes.thy \ |
|
612 Old_Number_Theory/WilsonBij.thy Old_Number_Theory/WilsonRuss.thy \ |
|
613 Old_Number_Theory/Finite2.thy Old_Number_Theory/Int2.thy \ |
|
614 Old_Number_Theory/EvenOdd.thy Old_Number_Theory/Residues.thy \ |
|
615 Old_Number_Theory/Euler.thy Old_Number_Theory/Gauss.thy \ |
|
616 Old_Number_Theory/Quadratic_Reciprocity.thy Library/Infinite_Set.thy \ |
|
617 Old_Number_Theory/Legacy_GCD.thy Old_Number_Theory/Pocklington.thy \ |
|
618 Old_Number_Theory/ROOT.ML |
|
619 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Old_Number_Theory |
|
620 |
|
621 |
|
622 ## HOL-Hoare |
|
623 |
|
624 HOL-Hoare: HOL $(LOG)/HOL-Hoare.gz |
|
625 |
|
626 $(LOG)/HOL-Hoare.gz: $(OUT)/HOL Hoare/Arith2.thy Hoare/Examples.thy \ |
|
627 Hoare/Hoare.thy Hoare/hoare_syntax.ML Hoare/hoare_tac.ML \ |
|
628 Hoare/Heap.thy Hoare/Hoare_Logic.thy Hoare/Hoare_Logic_Abort.thy \ |
|
629 Hoare/HeapSyntax.thy Hoare/Pointer_Examples.thy Hoare/ROOT.ML \ |
|
630 Hoare/ExamplesAbort.thy Hoare/HeapSyntaxAbort.thy \ |
|
631 Hoare/SchorrWaite.thy Hoare/Separation.thy Hoare/SepLogHeap.thy \ |
|
632 Hoare/document/root.tex Hoare/document/root.bib |
|
633 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Hoare |
|
634 |
|
635 |
|
636 ## HOL-Hoare_Parallel |
|
637 |
|
638 HOL-Hoare_Parallel: HOL $(LOG)/HOL-Hoare_Parallel.gz |
|
639 |
|
640 $(LOG)/HOL-Hoare_Parallel.gz: $(OUT)/HOL Hoare_Parallel/Gar_Coll.thy \ |
|
641 Hoare_Parallel/Graph.thy Hoare_Parallel/Hoare_Parallel.thy \ |
|
642 Hoare_Parallel/Mul_Gar_Coll.thy Hoare_Parallel/OG_Com.thy \ |
|
643 Hoare_Parallel/OG_Examples.thy Hoare_Parallel/OG_Hoare.thy \ |
|
644 Hoare_Parallel/OG_Syntax.thy Hoare_Parallel/OG_Tactics.thy \ |
|
645 Hoare_Parallel/OG_Tran.thy Hoare_Parallel/Quote_Antiquote.thy \ |
|
646 Hoare_Parallel/RG_Com.thy Hoare_Parallel/RG_Examples.thy \ |
|
647 Hoare_Parallel/RG_Hoare.thy Hoare_Parallel/RG_Syntax.thy \ |
|
648 Hoare_Parallel/RG_Tran.thy Hoare_Parallel/ROOT.ML \ |
|
649 Hoare_Parallel/document/root.tex Hoare_Parallel/document/root.bib |
|
650 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Hoare_Parallel |
|
651 |
|
652 |
|
653 ## HOL-Library-Codegenerator_Test |
|
654 |
|
655 HOL-Library-Codegenerator_Test: HOL-Library $(LOG)/HOL-Library-Codegenerator_Test.gz |
|
656 |
|
657 $(LOG)/HOL-Library-Codegenerator_Test.gz: $(OUT)/HOL-Library \ |
|
658 Codegenerator_Test/ROOT.ML \ |
|
659 Codegenerator_Test/Candidates.thy \ |
|
660 Codegenerator_Test/Candidates_Pretty.thy \ |
|
661 Codegenerator_Test/Generate.thy \ |
|
662 Codegenerator_Test/Generate_Pretty.thy |
|
663 @$(ISABELLE_TOOL) usedir -d false -g false -i false $(OUT)/HOL-Library Codegenerator_Test |
|
664 |
|
665 |
|
666 ## HOL-Metis_Examples |
|
667 |
|
668 HOL-Metis_Examples: HOL $(LOG)/HOL-Metis_Examples.gz |
|
669 |
|
670 $(LOG)/HOL-Metis_Examples.gz: $(OUT)/HOL Metis_Examples/ROOT.ML \ |
|
671 Metis_Examples/Abstraction.thy Metis_Examples/Big_O.thy \ |
|
672 Metis_Examples/Binary_Tree.thy Metis_Examples/Clausification.thy \ |
|
673 Metis_Examples/Message.thy Metis_Examples/Proxies.thy \ |
|
674 Metis_Examples/Sets.thy Metis_Examples/Tarski.thy \ |
|
675 Metis_Examples/Trans_Closure.thy Metis_Examples/Type_Encodings.thy |
|
676 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Metis_Examples |
|
677 |
|
678 |
|
679 ## HOL-Nitpick_Examples |
|
680 |
|
681 HOL-Nitpick_Examples: HOL $(LOG)/HOL-Nitpick_Examples.gz |
|
682 |
|
683 $(LOG)/HOL-Nitpick_Examples.gz: $(OUT)/HOL Nitpick_Examples/ROOT.ML \ |
|
684 Nitpick_Examples/Core_Nits.thy Nitpick_Examples/Datatype_Nits.thy \ |
|
685 Nitpick_Examples/Hotel_Nits.thy Nitpick_Examples/Induct_Nits.thy \ |
|
686 Nitpick_Examples/Integer_Nits.thy Nitpick_Examples/Manual_Nits.thy \ |
|
687 Nitpick_Examples/Mini_Nits.thy Nitpick_Examples/Mono_Nits.thy \ |
|
688 Nitpick_Examples/Nitpick_Examples.thy Nitpick_Examples/Pattern_Nits.thy \ |
|
689 Nitpick_Examples/Record_Nits.thy Nitpick_Examples/Refute_Nits.thy \ |
|
690 Nitpick_Examples/Special_Nits.thy Nitpick_Examples/Tests_Nits.thy \ |
|
691 Nitpick_Examples/Typedef_Nits.thy Nitpick_Examples/minipick.ML |
|
692 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Nitpick_Examples |
|
693 |
|
694 |
|
695 ## HOL-Algebra |
|
696 |
|
697 HOL-Algebra: HOL $(OUT)/HOL-Algebra |
|
698 |
|
699 ALGEBRA_DEPENDENCIES = $(OUT)/HOL \ |
|
700 Algebra/ROOT.ML \ |
|
701 Library/Binomial.thy \ |
|
702 Library/FuncSet.thy \ |
|
703 Library/Multiset.thy \ |
|
704 Library/Permutation.thy \ |
|
705 Number_Theory/Primes.thy \ |
|
706 Algebra/AbelCoset.thy \ |
|
707 Algebra/Bij.thy \ |
|
708 Algebra/Congruence.thy \ |
|
709 Algebra/Coset.thy \ |
|
710 Algebra/Divisibility.thy \ |
|
711 Algebra/Exponent.thy \ |
|
712 Algebra/FiniteProduct.thy \ |
|
713 Algebra/Group.thy \ |
|
714 Algebra/Ideal.thy \ |
|
715 Algebra/IntRing.thy \ |
|
716 Algebra/Lattice.thy \ |
|
717 Algebra/Module.thy \ |
|
718 Algebra/QuotRing.thy \ |
|
719 Algebra/Ring.thy \ |
|
720 Algebra/RingHom.thy \ |
|
721 Algebra/Sylow.thy \ |
|
722 Algebra/UnivPoly.thy \ |
|
723 Algebra/abstract/Abstract.thy \ |
|
724 Algebra/abstract/Factor.thy \ |
|
725 Algebra/abstract/Field.thy \ |
|
726 Algebra/abstract/Ideal2.thy \ |
|
727 Algebra/abstract/PID.thy \ |
|
728 Algebra/abstract/Ring2.thy \ |
|
729 Algebra/abstract/RingHomo.thy \ |
|
730 Algebra/document/root.tex \ |
|
731 Algebra/document/root.tex \ |
|
732 Algebra/poly/LongDiv.thy \ |
|
733 Algebra/poly/PolyHomo.thy \ |
|
734 Algebra/poly/Polynomial.thy \ |
|
735 Algebra/poly/UnivPoly2.thy \ |
|
736 Algebra/ringsimp.ML |
|
737 |
|
738 $(OUT)/HOL-Algebra: $(ALGEBRA_DEPENDENCIES) |
|
739 @cd Algebra; $(ISABELLE_TOOL) usedir -b -g true -V outline=/proof,/ML $(OUT)/HOL HOL-Algebra |
|
740 |
|
741 |
|
742 ## HOL-Auth |
|
743 |
|
744 HOL-Auth: HOL $(LOG)/HOL-Auth.gz |
|
745 |
|
746 $(LOG)/HOL-Auth.gz: $(OUT)/HOL \ |
|
747 Auth/Auth_Shared.thy Auth/Auth_Public.thy Auth/All_Symmetric.thy \ |
|
748 Auth/Guard/Auth_Guard_Shared.thy \ |
|
749 Auth/Guard/Auth_Guard_Public.thy \ |
|
750 Auth/Smartcard/Auth_Smartcard.thy Auth/All_Symmetric.thy \ |
|
751 Auth/CertifiedEmail.thy Auth/Event.thy Auth/Message.thy \ |
|
752 Auth/NS_Public.thy Auth/NS_Public_Bad.thy Auth/NS_Shared.thy \ |
|
753 Auth/OtwayRees.thy Auth/OtwayReesBella.thy Auth/OtwayRees_AN.thy \ |
|
754 Auth/OtwayRees_Bad.thy Auth/Public.thy Auth/ROOT.ML Auth/Recur.thy \ |
|
755 Auth/Shared.thy Auth/TLS.thy Auth/WooLam.thy Auth/Kerberos_BAN.thy \ |
|
756 Auth/Kerberos_BAN_Gets.thy Auth/KerberosIV.thy \ |
|
757 Auth/KerberosIV_Gets.thy Auth/KerberosV.thy Auth/Yahalom.thy \ |
|
758 Auth/Yahalom2.thy Auth/Yahalom_Bad.thy Auth/ZhouGollmann.thy \ |
|
759 Auth/Guard/Analz.thy Auth/Guard/Extensions.thy Auth/Guard/GuardK.thy \ |
|
760 Auth/Guard/Guard_Public.thy Auth/Guard/Guard_Shared.thy \ |
|
761 Auth/Guard/Guard.thy Auth/Guard/List_Msg.thy \ |
|
762 Auth/Guard/Guard_NS_Public.thy Auth/Guard/Guard_OtwayRees.thy \ |
|
763 Auth/Guard/P1.thy Auth/Guard/P2.thy Auth/Guard/Proto.thy \ |
|
764 Auth/Guard/Guard_Yahalom.thy Auth/Smartcard/EventSC.thy \ |
|
765 Auth/Smartcard/ShoupRubinBella.thy Auth/Smartcard/ShoupRubin.thy \ |
|
766 Auth/Smartcard/Smartcard.thy Auth/document/root.tex |
|
767 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Auth |
|
768 |
|
769 |
|
770 ## HOL-UNITY |
|
771 |
|
772 HOL-UNITY: HOL $(LOG)/HOL-UNITY.gz |
|
773 |
|
774 $(LOG)/HOL-UNITY.gz: $(OUT)/HOL Library/Multiset.thy UNITY/ROOT.ML \ |
|
775 UNITY/UNITY_Main.thy UNITY/UNITY_tactics.ML UNITY/Comp.thy \ |
|
776 UNITY/Constrains.thy UNITY/Detects.thy UNITY/ELT.thy \ |
|
777 UNITY/Extend.thy UNITY/FP.thy UNITY/Follows.thy UNITY/Guar.thy \ |
|
778 UNITY/Lift_prog.thy UNITY/ListOrder.thy UNITY/ProgressSets.thy \ |
|
779 UNITY/PPROD.thy UNITY/Project.thy UNITY/Rename.thy \ |
|
780 UNITY/Transformers.thy UNITY/SubstAx.thy UNITY/UNITY.thy \ |
|
781 UNITY/Union.thy UNITY/WFair.thy UNITY/Simple/Channel.thy \ |
|
782 UNITY/Simple/Common.thy UNITY/Simple/Deadlock.thy \ |
|
783 UNITY/Simple/Lift.thy UNITY/Simple/Mutex.thy \ |
|
784 UNITY/Simple/NSP_Bad.thy UNITY/Simple/Network.thy \ |
|
785 UNITY/Simple/Reach.thy UNITY/Simple/Reachability.thy \ |
|
786 UNITY/Simple/Token.thy UNITY/Comp/Alloc.thy UNITY/Comp/AllocBase.thy \ |
|
787 UNITY/Comp/AllocImpl.thy UNITY/Comp/Client.thy \ |
|
788 UNITY/Comp/Counter.thy UNITY/Comp/Counterc.thy \ |
|
789 UNITY/Comp/Handshake.thy UNITY/Comp/PriorityAux.thy \ |
|
790 UNITY/Comp/Priority.thy UNITY/Comp/Progress.thy \ |
|
791 UNITY/Comp/TimerArray.thy UNITY/document/root.tex |
|
792 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL UNITY |
|
793 |
|
794 |
|
795 ## HOL-Unix |
|
796 |
|
797 HOL-Unix: HOL $(LOG)/HOL-Unix.gz |
|
798 |
|
799 $(LOG)/HOL-Unix.gz: $(OUT)/HOL Library/List_Prefix.thy Unix/ROOT.ML \ |
|
800 Unix/Nested_Environment.thy Unix/Unix.thy Unix/document/root.bib \ |
|
801 Unix/document/root.tex |
|
802 @$(ISABELLE_TOOL) usedir -m no_brackets -m no_type_brackets $(OUT)/HOL Unix |
|
803 |
|
804 |
|
805 ## HOL-ZF |
|
806 |
|
807 HOL-ZF: HOL $(LOG)/HOL-ZF.gz |
|
808 |
|
809 $(LOG)/HOL-ZF.gz: $(OUT)/HOL ZF/ROOT.ML ZF/LProd.thy \ |
|
810 ZF/HOLZF.thy ZF/MainZF.thy ZF/Games.thy ZF/document/root.tex |
|
811 @$(ISABELLE_TOOL) usedir $(OUT)/HOL ZF |
|
812 |
|
813 |
|
814 ## HOL-Imperative_HOL |
|
815 |
|
816 HOL-Imperative_HOL: HOL $(LOG)/HOL-Imperative_HOL.gz |
|
817 |
|
818 $(LOG)/HOL-Imperative_HOL.gz: $(OUT)/HOL \ |
|
819 Library/Code_Integer.thy \ |
|
820 Library/Code_Nat.thy \ |
|
821 Library/Code_Natural.thy \ |
|
822 Library/Efficient_Nat.thy \ |
|
823 Imperative_HOL/Array.thy \ |
|
824 Imperative_HOL/Heap.thy \ |
|
825 Imperative_HOL/Heap_Monad.thy \ |
|
826 Imperative_HOL/Imperative_HOL.thy \ |
|
827 Imperative_HOL/Imperative_HOL_ex.thy \ |
|
828 Imperative_HOL/Mrec.thy \ |
|
829 Imperative_HOL/Ref.thy \ |
|
830 Imperative_HOL/ROOT.ML \ |
|
831 Imperative_HOL/ex/Imperative_Quicksort.thy \ |
|
832 Imperative_HOL/ex/Imperative_Reverse.thy \ |
|
833 Imperative_HOL/ex/Linked_Lists.thy \ |
|
834 Imperative_HOL/ex/SatChecker.thy \ |
|
835 Imperative_HOL/ex/Sorted_List.thy \ |
|
836 Imperative_HOL/ex/Subarray.thy \ |
|
837 Imperative_HOL/ex/Sublist.thy |
|
838 @$(ISABELLE_TOOL) usedir -g true -m iff -m no_brackets $(OUT)/HOL Imperative_HOL |
|
839 |
|
840 |
|
841 ## HOL-Decision_Procs |
|
842 |
|
843 HOL-Decision_Procs: HOL $(LOG)/HOL-Decision_Procs.gz |
|
844 |
|
845 $(LOG)/HOL-Decision_Procs.gz: $(OUT)/HOL \ |
|
846 Library/Code_Integer.thy \ |
|
847 Library/Code_Nat.thy \ |
|
848 Library/Code_Natural.thy \ |
|
849 Library/Efficient_Nat.thy \ |
|
850 Decision_Procs/Approximation.thy \ |
|
851 Decision_Procs/Commutative_Ring.thy \ |
|
852 Decision_Procs/Commutative_Ring_Complete.thy \ |
|
853 Decision_Procs/Cooper.thy \ |
|
854 Decision_Procs/Decision_Procs.thy \ |
|
855 Decision_Procs/Dense_Linear_Order.thy \ |
|
856 Decision_Procs/Ferrack.thy \ |
|
857 Decision_Procs/MIR.thy \ |
|
858 Decision_Procs/Parametric_Ferrante_Rackoff.thy \ |
|
859 Decision_Procs/Polynomial_List.thy \ |
|
860 Decision_Procs/ROOT.ML \ |
|
861 Decision_Procs/Reflected_Multivariate_Polynomial.thy \ |
|
862 Decision_Procs/commutative_ring_tac.ML \ |
|
863 Decision_Procs/cooper_tac.ML \ |
|
864 Decision_Procs/ex/Approximation_Ex.thy \ |
|
865 Decision_Procs/ex/Commutative_Ring_Ex.thy \ |
|
866 Decision_Procs/ex/Dense_Linear_Order_Ex.thy \ |
|
867 Decision_Procs/ferrack_tac.ML \ |
|
868 Decision_Procs/ferrante_rackoff.ML \ |
|
869 Decision_Procs/ferrante_rackoff_data.ML \ |
|
870 Decision_Procs/langford.ML \ |
|
871 Decision_Procs/langford_data.ML \ |
|
872 Decision_Procs/mir_tac.ML |
|
873 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Decision_Procs |
|
874 |
|
875 |
|
876 ## HOL-Proofs |
|
877 |
|
878 HOL-Proofs: Pure $(OUT)/HOL-Proofs |
|
879 |
|
880 $(OUT)/HOL-Proofs: main.ML $(MAIN_DEPENDENCIES) |
|
881 @$(ISABELLE_TOOL) usedir -b -f main.ML -g true -p 2 -q 0 $(OUT)/Pure HOL-Proofs |
|
882 |
|
883 |
|
884 ## HOL-Proofs-ex |
|
885 |
|
886 HOL-Proofs-ex: HOL-Proofs $(LOG)/HOL-Proofs-ex.gz |
|
887 |
|
888 $(LOG)/HOL-Proofs-ex.gz: $(OUT)/HOL-Proofs \ |
|
889 Proofs/ex/ROOT.ML Proofs/ex/Hilbert_Classical.thy |
|
890 @cd Proofs; $(ISABELLE_TOOL) usedir -p 2 -q 0 $(OUT)/HOL-Proofs ex |
|
891 |
|
892 |
|
893 ## HOL-Proofs-Extraction |
|
894 |
|
895 HOL-Proofs-Extraction: HOL-Proofs $(LOG)/HOL-Proofs-Extraction.gz |
|
896 |
|
897 $(LOG)/HOL-Proofs-Extraction.gz: $(OUT)/HOL-Proofs \ |
|
898 Library/Code_Integer.thy Library/Code_Nat.thy \ |
|
899 Library/Code_Natural.thy Library/Efficient_Nat.thy \ |
|
900 Proofs/Extraction/Euclid.thy \ |
|
901 Proofs/Extraction/Greatest_Common_Divisor.thy \ |
|
902 Proofs/Extraction/Higman.thy \ |
|
903 Proofs/Extraction/Higman_Extraction.thy \ |
|
904 Proofs/Extraction/Pigeonhole.thy \ |
|
905 Proofs/Extraction/QuotRem.thy Proofs/Extraction/ROOT.ML \ |
|
906 Proofs/Extraction/Util.thy Proofs/Extraction/Warshall.thy \ |
|
907 Proofs/Extraction/document/root.tex \ |
|
908 Proofs/Extraction/document/root.bib |
|
909 @cd Proofs; $(ISABELLE_TOOL) usedir -p 2 -q 0 $(OUT)/HOL-Proofs Extraction |
|
910 |
|
911 |
|
912 ## HOL-Proofs-Lambda |
|
913 |
|
914 HOL-Proofs-Lambda: HOL-Proofs $(LOG)/HOL-Proofs-Lambda.gz |
|
915 |
|
916 $(LOG)/HOL-Proofs-Lambda.gz: $(OUT)/HOL-Proofs \ |
|
917 Proofs/Lambda/Commutation.thy Proofs/Lambda/Eta.thy \ |
|
918 Proofs/Lambda/InductTermi.thy Proofs/Lambda/Lambda.thy \ |
|
919 Proofs/Lambda/ListApplication.thy Proofs/Lambda/ListBeta.thy \ |
|
920 Proofs/Lambda/ListOrder.thy Proofs/Lambda/NormalForm.thy \ |
|
921 Proofs/Lambda/ParRed.thy Proofs/Lambda/Standardization.thy \ |
|
922 Proofs/Lambda/StrongNorm.thy Proofs/Lambda/Type.thy \ |
|
923 Proofs/Lambda/WeakNorm.thy Proofs/Lambda/ROOT.ML \ |
|
924 Proofs/Lambda/document/root.bib Proofs/Lambda/document/root.tex |
|
925 @cd Proofs; $(ISABELLE_TOOL) usedir -g true -m no_brackets -p 2 -q 0 $(OUT)/HOL-Proofs Lambda |
|
926 |
|
927 |
|
928 ## HOL-Prolog |
|
929 |
|
930 HOL-Prolog: HOL $(LOG)/HOL-Prolog.gz |
|
931 |
|
932 $(LOG)/HOL-Prolog.gz: $(OUT)/HOL Prolog/ROOT.ML Prolog/prolog.ML \ |
|
933 Prolog/HOHH.thy Prolog/Test.thy Prolog/Func.thy Prolog/Type.thy |
|
934 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Prolog |
|
935 |
|
936 |
|
937 ## HOL-MicroJava |
|
938 |
|
939 HOL-MicroJava: HOL $(LOG)/HOL-MicroJava.gz |
|
940 |
|
941 $(LOG)/HOL-MicroJava.gz: $(OUT)/HOL MicroJava/ROOT.ML \ |
|
942 MicroJava/Comp/AuxLemmas.thy MicroJava/Comp/CorrComp.thy \ |
|
943 MicroJava/Comp/CorrCompTp.thy MicroJava/Comp/DefsComp.thy \ |
|
944 MicroJava/Comp/Index.thy MicroJava/Comp/LemmasComp.thy \ |
|
945 MicroJava/Comp/TranslComp.thy MicroJava/Comp/TranslCompTp.thy \ |
|
946 MicroJava/Comp/TypeInf.thy MicroJava/J/Conform.thy \ |
|
947 MicroJava/J/Eval.thy MicroJava/J/JBasis.thy \ |
|
948 MicroJava/J/JTypeSafe.thy MicroJava/J/Decl.thy MicroJava/J/State.thy \ |
|
949 MicroJava/J/Term.thy MicroJava/J/Type.thy MicroJava/J/TypeRel.thy \ |
|
950 MicroJava/J/WellForm.thy MicroJava/J/Value.thy \ |
|
951 MicroJava/J/WellType.thy MicroJava/J/Example.thy \ |
|
952 MicroJava/J/JListExample.thy MicroJava/JVM/JVMExec.thy \ |
|
953 MicroJava/JVM/JVMInstructions.thy MicroJava/JVM/JVMState.thy \ |
|
954 MicroJava/JVM/JVMExecInstr.thy MicroJava/JVM/JVMListExample.thy \ |
|
955 MicroJava/JVM/JVMExceptions.thy MicroJava/DFA/Abstract_BV.thy \ |
|
956 MicroJava/DFA/Err.thy MicroJava/DFA/Kildall.thy \ |
|
957 MicroJava/DFA/LBVComplete.thy MicroJava/DFA/LBVCorrect.thy \ |
|
958 MicroJava/DFA/LBVSpec.thy MicroJava/DFA/Listn.thy \ |
|
959 MicroJava/DFA/Opt.thy MicroJava/DFA/Product.thy \ |
|
960 MicroJava/DFA/SemilatAlg.thy MicroJava/DFA/Semilat.thy \ |
|
961 MicroJava/DFA/Semilattices.thy \ |
|
962 MicroJava/DFA/Typing_Framework_err.thy \ |
|
963 MicroJava/DFA/Typing_Framework.thy MicroJava/BV/BVSpec.thy \ |
|
964 MicroJava/BV/BVSpecTypeSafe.thy MicroJava/BV/Correct.thy \ |
|
965 MicroJava/BV/JType.thy MicroJava/BV/JVM.thy MicroJava/BV/JVMType.thy \ |
|
966 MicroJava/BV/Effect.thy MicroJava/BV/EffectMono.thy \ |
|
967 MicroJava/BV/Typing_Framework_JVM.thy MicroJava/BV/BVExample.thy \ |
|
968 MicroJava/BV/LBVJVM.thy MicroJava/document/root.bib \ |
|
969 MicroJava/document/root.tex MicroJava/document/introduction.tex |
|
970 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL MicroJava |
|
971 |
|
972 |
|
973 ## HOL-NanoJava |
|
974 |
|
975 HOL-NanoJava: HOL $(LOG)/HOL-NanoJava.gz |
|
976 |
|
977 $(LOG)/HOL-NanoJava.gz: $(OUT)/HOL NanoJava/ROOT.ML NanoJava/Term.thy \ |
|
978 NanoJava/Decl.thy NanoJava/TypeRel.thy NanoJava/State.thy \ |
|
979 NanoJava/OpSem.thy NanoJava/AxSem.thy NanoJava/AxSem.thy \ |
|
980 NanoJava/document/root.bib NanoJava/document/root.tex |
|
981 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL NanoJava |
|
982 |
|
983 |
|
984 ## HOL-Bali |
|
985 |
|
986 HOL-Bali: HOL $(LOG)/HOL-Bali.gz |
|
987 |
|
988 $(LOG)/HOL-Bali.gz: $(OUT)/HOL Bali/AxCompl.thy Bali/AxExample.thy \ |
|
989 Bali/AxSem.thy Bali/AxSound.thy Bali/Basis.thy Bali/Conform.thy \ |
|
990 Bali/Decl.thy Bali/DeclConcepts.thy Bali/Eval.thy Bali/Evaln.thy \ |
|
991 Bali/Example.thy Bali/Name.thy Bali/ROOT.ML Bali/State.thy \ |
|
992 Bali/Table.thy Bali/Term.thy Bali/Trans.thy Bali/Type.thy \ |
|
993 Bali/TypeRel.thy Bali/TypeSafe.thy Bali/Value.thy Bali/WellForm.thy \ |
|
994 Bali/DefiniteAssignment.thy Bali/DefiniteAssignmentCorrect.thy \ |
|
995 Bali/WellType.thy Bali/document/root.tex |
|
996 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Bali |
|
997 |
|
998 |
|
999 ## HOL-IOA |
|
1000 |
|
1001 HOL-IOA: HOL $(LOG)/HOL-IOA.gz |
|
1002 |
|
1003 $(LOG)/HOL-IOA.gz: $(OUT)/HOL IOA/Asig.thy IOA/IOA.thy IOA/ROOT.ML \ |
|
1004 IOA/Solve.thy |
|
1005 @$(ISABELLE_TOOL) usedir $(OUT)/HOL IOA |
|
1006 |
|
1007 |
|
1008 ## HOL-Lattice |
|
1009 |
|
1010 HOL-Lattice: HOL $(LOG)/HOL-Lattice.gz |
|
1011 |
|
1012 $(LOG)/HOL-Lattice.gz: $(OUT)/HOL Lattice/Bounds.thy \ |
|
1013 Lattice/CompleteLattice.thy Lattice/Lattice.thy Lattice/Orders.thy \ |
|
1014 Lattice/ROOT.ML Lattice/document/root.tex |
|
1015 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Lattice |
|
1016 |
|
1017 |
|
1018 ## HOL-ex |
|
1019 |
|
1020 HOL-ex: HOL $(LOG)/HOL-ex.gz |
|
1021 |
|
1022 $(LOG)/HOL-ex.gz: $(OUT)/HOL Decision_Procs/Commutative_Ring.thy \ |
|
1023 Library/Code_Integer.thy Library/Code_Nat.thy \ |
|
1024 Library/Code_Natural.thy Library/Efficient_Nat.thy \ |
|
1025 Number_Theory/Primes.thy ex/Abstract_NAT.thy ex/Antiquote.thy \ |
|
1026 ex/Arith_Examples.thy ex/BT.thy \ |
|
1027 ex/BinEx.thy ex/Binary.thy ex/Birthday_Paradox.thy ex/CTL.thy \ |
|
1028 ex/Case_Product.thy ex/Chinese.thy ex/Classical.thy \ |
|
1029 ex/Code_Nat_examples.thy \ |
|
1030 ex/Coercion_Examples.thy ex/Coherent.thy ex/Dedekind_Real.thy \ |
|
1031 ex/Eval_Examples.thy ex/Executable_Relation.thy \ |
|
1032 ex/FinFunPred.thy ex/Fundefs.thy \ |
|
1033 ex/Gauge_Integration.thy ex/Groebner_Examples.thy ex/Guess.thy \ |
|
1034 ex/HarmonicSeries.thy ex/Hebrew.thy ex/Hex_Bin_Examples.thy \ |
|
1035 ex/Higher_Order_Logic.thy ex/Iff_Oracle.thy ex/Induction_Schema.thy \ |
|
1036 ex/Interpretation_with_Defs.thy ex/Intuitionistic.thy \ |
|
1037 ex/Lagrange.thy ex/List_to_Set_Comprehension_Examples.thy \ |
|
1038 ex/LocaleTest2.thy ex/MT.thy ex/MergeSort.thy ex/Meson_Test.thy \ |
|
1039 ex/MonoidGroup.thy ex/Multiquote.thy ex/NatSum.thy \ |
|
1040 ex/Normalization_by_Evaluation.thy ex/Numeral_Representation.thy \ |
|
1041 ex/Parallel_Example.thy \ |
|
1042 ex/PER.thy ex/PresburgerEx.thy ex/Primrec.thy \ |
|
1043 ex/Quicksort.thy ex/ROOT.ML \ |
|
1044 ex/Records.thy ex/ReflectionEx.thy ex/Refute_Examples.thy \ |
|
1045 ex/SAT_Examples.thy ex/Serbian.thy \ |
|
1046 ex/Set_Comprehension_Pointfree_Tests.thy ex/Set_Theory.thy \ |
|
1047 ex/Simproc_Tests.thy ex/SVC_Oracle.thy \ |
|
1048 ex/Seq.thy ex/Sqrt.thy ex/Sqrt_Script.thy \ |
|
1049 ex/Sudoku.thy ex/Tarski.thy ex/Termination.thy ex/Transfer_Ex.thy \ |
|
1050 ex/Transfer_Int_Nat.thy \ |
|
1051 ex/Tree23.thy ex/Unification.thy ex/While_Combinator_Example.thy \ |
|
1052 ex/document/root.bib ex/document/root.tex ex/svc_funcs.ML \ |
|
1053 ex/svc_test.thy ../Tools/interpretation_with_defs.ML |
|
1054 @$(ISABELLE_TOOL) usedir $(OUT)/HOL ex |
|
1055 |
|
1056 |
|
1057 ## HOL-Isar_Examples |
|
1058 |
|
1059 HOL-Isar_Examples: HOL $(LOG)/HOL-Isar_Examples.gz |
|
1060 |
|
1061 $(LOG)/HOL-Isar_Examples.gz: $(OUT)/HOL Isar_Examples/Basic_Logic.thy \ |
|
1062 Isar_Examples/Cantor.thy Isar_Examples/Drinker.thy \ |
|
1063 Isar_Examples/Expr_Compiler.thy Isar_Examples/Fibonacci.thy \ |
|
1064 Isar_Examples/Group.thy Isar_Examples/Group_Context.thy \ |
|
1065 Isar_Examples/Group_Notepad.thy Isar_Examples/Hoare.thy \ |
|
1066 Isar_Examples/Hoare_Ex.thy Isar_Examples/Knaster_Tarski.thy \ |
|
1067 Isar_Examples/Mutilated_Checkerboard.thy \ |
|
1068 Isar_Examples/Nested_Datatype.thy Isar_Examples/Peirce.thy \ |
|
1069 Isar_Examples/Puzzle.thy Isar_Examples/Summation.thy \ |
|
1070 Isar_Examples/ROOT.ML Isar_Examples/document/proof.sty \ |
|
1071 Isar_Examples/document/root.bib Isar_Examples/document/root.tex \ |
|
1072 Isar_Examples/document/style.tex Hoare/hoare_tac.ML \ |
|
1073 Number_Theory/Primes.thy |
|
1074 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Isar_Examples |
|
1075 |
|
1076 |
|
1077 ## HOL-SET_Protocol |
|
1078 |
|
1079 HOL-SET_Protocol: HOL $(LOG)/HOL-SET_Protocol.gz |
|
1080 |
|
1081 $(LOG)/HOL-SET_Protocol.gz: $(OUT)/HOL SET_Protocol/ROOT.ML \ |
|
1082 SET_Protocol/Message_SET.thy SET_Protocol/Event_SET.thy \ |
|
1083 SET_Protocol/Public_SET.thy SET_Protocol/Cardholder_Registration.thy \ |
|
1084 SET_Protocol/Merchant_Registration.thy SET_Protocol/Purchase.thy \ |
|
1085 SET_Protocol/SET_Protocol.thy SET_Protocol/document/root.tex |
|
1086 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL SET_Protocol |
|
1087 |
|
1088 |
|
1089 ## HOL-Matrix_LP |
|
1090 |
|
1091 HOL-Matrix_LP: HOL $(LOG)/HOL-Matrix_LP.gz |
|
1092 |
|
1093 $(LOG)/HOL-Matrix_LP.gz: $(OUT)/HOL Matrix_LP/ComputeFloat.thy \ |
|
1094 Matrix_LP/ComputeHOL.thy Matrix_LP/ComputeNumeral.thy \ |
|
1095 Matrix_LP/Compute_Oracle/Compute_Oracle.thy \ |
|
1096 Matrix_LP/Compute_Oracle/am.ML \ |
|
1097 Matrix_LP/Compute_Oracle/am_compiler.ML \ |
|
1098 Matrix_LP/Compute_Oracle/am_ghc.ML \ |
|
1099 Matrix_LP/Compute_Oracle/am_interpreter.ML \ |
|
1100 Matrix_LP/Compute_Oracle/am_sml.ML \ |
|
1101 Matrix_LP/Compute_Oracle/compute.ML \ |
|
1102 Matrix_LP/Compute_Oracle/linker.ML Matrix_LP/Cplex.thy \ |
|
1103 Matrix_LP/CplexMatrixConverter.ML Matrix_LP/Cplex_tools.ML \ |
|
1104 Matrix_LP/FloatSparseMatrixBuilder.ML Matrix_LP/LP.thy \ |
|
1105 Matrix_LP/Matrix.thy Matrix_LP/ROOT.ML Matrix_LP/SparseMatrix.thy \ |
|
1106 Matrix_LP/document/root.tex Matrix_LP/fspmlp.ML \ |
|
1107 Matrix_LP/matrixlp.ML Tools/float_arith.ML |
|
1108 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Matrix_LP |
|
1109 |
|
1110 |
|
1111 ## TLA |
|
1112 |
|
1113 TLA: HOL $(OUT)/TLA |
|
1114 |
|
1115 $(OUT)/TLA: $(OUT)/HOL TLA/Action.thy TLA/Init.thy TLA/Intensional.thy \ |
|
1116 TLA/ROOT.ML TLA/Stfun.thy TLA/TLA.thy |
|
1117 @cd TLA; $(ISABELLE_TOOL) usedir -b $(OUT)/HOL TLA |
|
1118 |
|
1119 |
|
1120 ## TLA-Inc |
|
1121 |
|
1122 TLA-Inc: TLA $(LOG)/TLA-Inc.gz |
|
1123 |
|
1124 $(LOG)/TLA-Inc.gz: $(OUT)/TLA TLA/Inc/Inc.thy |
|
1125 @cd TLA; $(ISABELLE_TOOL) usedir $(OUT)/TLA Inc |
|
1126 |
|
1127 |
|
1128 ## TLA-Buffer |
|
1129 |
|
1130 TLA-Buffer: TLA $(LOG)/TLA-Buffer.gz |
|
1131 |
|
1132 $(LOG)/TLA-Buffer.gz: $(OUT)/TLA TLA/Buffer/Buffer.thy \ |
|
1133 TLA/Buffer/DBuffer.thy |
|
1134 @cd TLA; $(ISABELLE_TOOL) usedir $(OUT)/TLA Buffer |
|
1135 |
|
1136 |
|
1137 ## TLA-Memory |
|
1138 |
|
1139 TLA-Memory: TLA $(LOG)/TLA-Memory.gz |
|
1140 |
|
1141 $(LOG)/TLA-Memory.gz: $(OUT)/TLA TLA/Memory/MemClerk.thy \ |
|
1142 TLA/Memory/MemClerkParameters.thy TLA/Memory/Memory.thy \ |
|
1143 TLA/Memory/MemoryImplementation.thy TLA/Memory/MemoryParameters.thy \ |
|
1144 TLA/Memory/ProcedureInterface.thy TLA/Memory/RPC.thy \ |
|
1145 TLA/Memory/RPCMemoryParams.thy TLA/Memory/RPCParameters.thy |
|
1146 @cd TLA; $(ISABELLE_TOOL) usedir $(OUT)/TLA Memory |
|
1147 |
|
1148 |
|
1149 ## HOL-TPTP |
|
1150 |
|
1151 HOL-TPTP: HOL $(LOG)/HOL-TPTP.gz |
|
1152 |
|
1153 $(LOG)/HOL-TPTP.gz: $(OUT)/HOL \ |
|
1154 TPTP/ATP_Problem_Import.thy \ |
|
1155 TPTP/ATP_Theory_Export.thy \ |
|
1156 TPTP/MaSh_Eval.thy \ |
|
1157 TPTP/MaSh_Export.thy \ |
|
1158 TPTP/ROOT.ML \ |
|
1159 TPTP/THF_Arith.thy \ |
|
1160 TPTP/TPTP_Parser.thy \ |
|
1161 TPTP/TPTP_Parser/ml_yacc_lib.ML \ |
|
1162 TPTP/TPTP_Parser/tptp_interpret.ML \ |
|
1163 TPTP/TPTP_Parser/tptp_lexyacc.ML \ |
|
1164 TPTP/TPTP_Parser/tptp_parser.ML \ |
|
1165 TPTP/TPTP_Parser/tptp_problem_name.ML \ |
|
1166 TPTP/TPTP_Parser/tptp_syntax.ML \ |
|
1167 TPTP/TPTP_Parser_Test.thy \ |
|
1168 TPTP/atp_problem_import.ML \ |
|
1169 TPTP/atp_theory_export.ML \ |
|
1170 TPTP/mash_eval.ML \ |
|
1171 TPTP/mash_export.ML \ |
|
1172 TPTP/sledgehammer_tactics.ML |
|
1173 @$(ISABELLE_TOOL) usedir $(OUT)/HOL TPTP |
|
1174 |
|
1175 |
|
1176 ## HOL-Multivariate_Analysis |
|
1177 |
|
1178 HOL-Multivariate_Analysis: HOL $(OUT)/HOL-Multivariate_Analysis |
|
1179 |
|
1180 $(OUT)/HOL-Multivariate_Analysis: $(OUT)/HOL \ |
|
1181 Multivariate_Analysis/Brouwer_Fixpoint.thy \ |
|
1182 Multivariate_Analysis/Cartesian_Euclidean_Space.thy \ |
|
1183 Multivariate_Analysis/Convex_Euclidean_Space.thy \ |
|
1184 Multivariate_Analysis/Derivative.thy \ |
|
1185 Multivariate_Analysis/Determinants.thy \ |
|
1186 Multivariate_Analysis/Euclidean_Space.thy \ |
|
1187 Multivariate_Analysis/Extended_Real_Limits.thy \ |
|
1188 Multivariate_Analysis/Fashoda.thy \ |
|
1189 Multivariate_Analysis/Finite_Cartesian_Product.thy \ |
|
1190 Multivariate_Analysis/Integration.certs \ |
|
1191 Multivariate_Analysis/Integration.thy \ |
|
1192 Multivariate_Analysis/L2_Norm.thy \ |
|
1193 Multivariate_Analysis/Linear_Algebra.thy \ |
|
1194 Multivariate_Analysis/Multivariate_Analysis.thy \ |
|
1195 Multivariate_Analysis/Norm_Arith.thy \ |
|
1196 Multivariate_Analysis/Operator_Norm.thy \ |
|
1197 Multivariate_Analysis/Path_Connected.thy \ |
|
1198 Multivariate_Analysis/ROOT.ML \ |
|
1199 Multivariate_Analysis/Real_Integration.thy \ |
|
1200 Multivariate_Analysis/Topology_Euclidean_Space.thy \ |
|
1201 Multivariate_Analysis/document/root.tex \ |
|
1202 Multivariate_Analysis/normarith.ML Library/Glbs.thy \ |
|
1203 Library/Extended_Real.thy Library/Indicator_Function.thy \ |
|
1204 Library/Inner_Product.thy Library/Numeral_Type.thy Library/Convex.thy \ |
|
1205 Library/FrechetDeriv.thy Library/Product_Vector.thy \ |
|
1206 Library/Product_plus.thy Library/Sum_of_Squares.thy |
|
1207 @cd Multivariate_Analysis; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL HOL-Multivariate_Analysis |
|
1208 |
|
1209 |
|
1210 ## HOL-Probability |
|
1211 |
|
1212 HOL-Probability: HOL-Multivariate_Analysis $(OUT)/HOL-Probability |
|
1213 |
|
1214 $(OUT)/HOL-Probability: $(OUT)/HOL-Multivariate_Analysis \ |
|
1215 Probability/Binary_Product_Measure.thy Probability/Borel_Space.thy \ |
|
1216 Probability/Caratheodory.thy Probability/Complete_Measure.thy \ |
|
1217 Probability/ex/Dining_Cryptographers.thy \ |
|
1218 Probability/ex/Koepf_Duermuth_Countermeasure.thy \ |
|
1219 Probability/Finite_Product_Measure.thy \ |
|
1220 Probability/Independent_Family.thy \ |
|
1221 Probability/Infinite_Product_Measure.thy Probability/Information.thy \ |
|
1222 Probability/Lebesgue_Integration.thy Probability/Lebesgue_Measure.thy \ |
|
1223 Probability/Measure_Space.thy Probability/Probability_Measure.thy \ |
|
1224 Probability/Probability.thy Probability/Radon_Nikodym.thy \ |
|
1225 Probability/ROOT.ML Probability/Sigma_Algebra.thy \ |
|
1226 Library/Countable.thy Library/FuncSet.thy Library/Nat_Bijection.thy |
|
1227 @cd Probability; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL-Multivariate_Analysis HOL-Probability |
|
1228 |
|
1229 |
|
1230 ## HOL-Nominal |
|
1231 |
|
1232 HOL-Nominal: HOL $(OUT)/HOL-Nominal |
|
1233 |
|
1234 $(OUT)/HOL-Nominal: $(OUT)/HOL Nominal/ROOT.ML \ |
|
1235 Nominal/Nominal.thy \ |
|
1236 Nominal/nominal_atoms.ML \ |
|
1237 Nominal/nominal_datatype.ML \ |
|
1238 Nominal/nominal_fresh_fun.ML \ |
|
1239 Nominal/nominal_induct.ML \ |
|
1240 Nominal/nominal_inductive.ML \ |
|
1241 Nominal/nominal_inductive2.ML \ |
|
1242 Nominal/nominal_permeq.ML \ |
|
1243 Nominal/nominal_primrec.ML \ |
|
1244 Nominal/nominal_thmdecls.ML \ |
|
1245 Library/Infinite_Set.thy |
|
1246 @cd Nominal; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL HOL-Nominal |
|
1247 |
|
1248 |
|
1249 ## HOL-Nominal-Examples |
|
1250 |
|
1251 HOL-Nominal-Examples: HOL-Nominal $(LOG)/HOL-Nominal-Examples.gz |
|
1252 |
|
1253 $(LOG)/HOL-Nominal-Examples.gz: $(OUT)/HOL-Nominal \ |
|
1254 Nominal/Examples/Nominal_Examples.thy \ |
|
1255 Nominal/Examples/CK_Machine.thy \ |
|
1256 Nominal/Examples/CR.thy \ |
|
1257 Nominal/Examples/CR_Takahashi.thy \ |
|
1258 Nominal/Examples/Class1.thy \ |
|
1259 Nominal/Examples/Class2.thy \ |
|
1260 Nominal/Examples/Class3.thy \ |
|
1261 Nominal/Examples/Compile.thy \ |
|
1262 Nominal/Examples/Contexts.thy \ |
|
1263 Nominal/Examples/Crary.thy \ |
|
1264 Nominal/Examples/Fsub.thy \ |
|
1265 Nominal/Examples/Height.thy \ |
|
1266 Nominal/Examples/Lam_Funs.thy \ |
|
1267 Nominal/Examples/Lambda_mu.thy \ |
|
1268 Nominal/Examples/LocalWeakening.thy \ |
|
1269 Nominal/Examples/Pattern.thy \ |
|
1270 Nominal/Examples/ROOT.ML \ |
|
1271 Nominal/Examples/SN.thy \ |
|
1272 Nominal/Examples/SOS.thy \ |
|
1273 Nominal/Examples/Standardization.thy \ |
|
1274 Nominal/Examples/Support.thy \ |
|
1275 Nominal/Examples/Type_Preservation.thy \ |
|
1276 Nominal/Examples/VC_Condition.thy \ |
|
1277 Nominal/Examples/W.thy \ |
|
1278 Nominal/Examples/Weakening.thy |
|
1279 @cd Nominal; $(ISABELLE_TOOL) usedir $(OUT)/HOL-Nominal Examples |
|
1280 |
|
1281 |
|
1282 ## HOL-Word |
|
1283 |
|
1284 HOL-Word: HOL $(OUT)/HOL-Word |
|
1285 |
|
1286 $(OUT)/HOL-Word: $(OUT)/HOL Word/ROOT.ML Library/Boolean_Algebra.thy \ |
|
1287 Library/Numeral_Type.thy Word/Misc_Numeric.thy Word/Misc_Typedef.thy \ |
|
1288 Word/Type_Length.thy Word/Bit_Representation.thy Word/Bit_Int.thy \ |
|
1289 Word/Bool_List_Representation.thy Word/Bit_Operations.thy \ |
|
1290 Word/Word.thy Word/WordBitwise.thy Word/document/root.tex \ |
|
1291 Word/document/root.bib Word/Tools/smt_word.ML Word/Tools/word_lib.ML |
|
1292 @cd Word; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL HOL-Word |
|
1293 |
|
1294 |
|
1295 ## HOL-Word-Examples |
|
1296 |
|
1297 HOL-Word-Examples: HOL-Word $(LOG)/HOL-Word-Examples.gz |
|
1298 |
|
1299 $(LOG)/HOL-Word-Examples.gz: $(OUT)/HOL-Word Word/Examples/ROOT.ML \ |
|
1300 Word/Examples/WordExamples.thy |
|
1301 @cd Word; $(ISABELLE_TOOL) usedir $(OUT)/HOL-Word Examples |
|
1302 |
|
1303 |
|
1304 ## HOL-Statespace |
|
1305 |
|
1306 HOL-Statespace: HOL $(LOG)/HOL-Statespace.gz |
|
1307 |
|
1308 $(LOG)/HOL-Statespace.gz: $(OUT)/HOL Statespace/ROOT.ML \ |
|
1309 Statespace/DistinctTreeProver.thy Statespace/StateFun.thy \ |
|
1310 Statespace/StateSpaceLocale.thy Statespace/StateSpaceSyntax.thy \ |
|
1311 Statespace/StateSpaceEx.thy Statespace/distinct_tree_prover.ML \ |
|
1312 Statespace/state_space.ML Statespace/state_fun.ML \ |
|
1313 Statespace/document/root.tex |
|
1314 @$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Statespace |
|
1315 |
|
1316 |
|
1317 ## HOL-NSA |
|
1318 |
|
1319 HOL-NSA: HOL $(OUT)/HOL-NSA |
|
1320 |
|
1321 $(OUT)/HOL-NSA: $(OUT)/HOL NSA/CLim.thy NSA/CStar.thy NSA/NSCA.thy \ |
|
1322 NSA/NSComplex.thy NSA/HDeriv.thy NSA/HLim.thy NSA/HLog.thy \ |
|
1323 NSA/HSEQ.thy NSA/HSeries.thy NSA/HTranscendental.thy \ |
|
1324 NSA/Hypercomplex.thy NSA/HyperDef.thy NSA/HyperNat.thy \ |
|
1325 NSA/Hyperreal.thy NSA/Filter.thy NSA/NatStar.thy NSA/NSA.thy \ |
|
1326 NSA/StarDef.thy NSA/Star.thy NSA/transfer.ML \ |
|
1327 Library/Infinite_Set.thy Library/Zorn.thy NSA/ROOT.ML |
|
1328 @cd NSA; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL HOL-NSA |
|
1329 |
|
1330 |
|
1331 ## HOL-NSA-Examples |
|
1332 |
|
1333 HOL-NSA-Examples: HOL-NSA $(LOG)/HOL-NSA-Examples.gz |
|
1334 |
|
1335 $(LOG)/HOL-NSA-Examples.gz: $(OUT)/HOL-NSA NSA/Examples/ROOT.ML \ |
|
1336 NSA/Examples/NSPrimes.thy |
|
1337 @cd NSA; $(ISABELLE_TOOL) usedir $(OUT)/HOL-NSA Examples |
|
1338 |
|
1339 |
|
1340 ## HOL-Mirabelle |
|
1341 |
|
1342 HOL-Mirabelle: HOL $(LOG)/HOL-Mirabelle.gz |
|
1343 |
|
1344 $(LOG)/HOL-Mirabelle.gz: $(OUT)/HOL Mirabelle/Mirabelle_Test.thy \ |
|
1345 Mirabelle/Mirabelle.thy Mirabelle/Tools/mirabelle.ML \ |
|
1346 Mirabelle/ROOT.ML Mirabelle/Tools/mirabelle_arith.ML \ |
|
1347 Mirabelle/Tools/mirabelle_metis.ML \ |
|
1348 Mirabelle/Tools/mirabelle_quickcheck.ML \ |
|
1349 Mirabelle/Tools/mirabelle_refute.ML \ |
|
1350 Mirabelle/Tools/mirabelle_sledgehammer.ML \ |
|
1351 Mirabelle/Tools/mirabelle_sledgehammer_filter.ML \ |
|
1352 Mirabelle/Tools/mirabelle_try0.ML \ |
|
1353 TPTP/sledgehammer_tactics.ML Mirabelle/lib/Tools/mirabelle \ |
|
1354 Mirabelle/lib/scripts/mirabelle.pl Library/FrechetDeriv.thy \ |
|
1355 Library/Inner_Product.thy |
|
1356 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Mirabelle |
|
1357 @cd Library; $(ISABELLE_TOOL) mirabelle -q arith Inner_Product.thy # some arbitrary small test case |
|
1358 |
|
1359 |
|
1360 ## HOL-Word-SMT_Examples |
|
1361 |
|
1362 HOL-Word-SMT_Examples: HOL-Word $(LOG)/HOL-Word-SMT_Examples.gz |
|
1363 |
|
1364 $(LOG)/HOL-Word-SMT_Examples.gz: $(OUT)/HOL-Word SMT_Examples/ROOT.ML \ |
|
1365 SMT_Examples/SMT_Examples.thy SMT_Examples/SMT_Examples.certs \ |
|
1366 SMT_Examples/SMT_Word_Examples.thy SMT_Examples/SMT_Tests.thy \ |
|
1367 SMT_Examples/SMT_Word_Examples.certs SMT_Examples/SMT_Tests.certs |
|
1368 @$(ISABELLE_TOOL) usedir $(OUT)/HOL-Word SMT_Examples |
|
1369 |
|
1370 |
|
1371 ## HOL-Boogie |
|
1372 |
|
1373 HOL-Boogie: HOL-Word $(OUT)/HOL-Boogie |
|
1374 |
|
1375 $(OUT)/HOL-Boogie: $(OUT)/HOL-Word Boogie/ROOT.ML Boogie/Boogie.thy \ |
|
1376 Boogie/Tools/boogie_vcs.ML Boogie/Tools/boogie_loader.ML \ |
|
1377 Boogie/Tools/boogie_commands.ML Boogie/Tools/boogie_tactics.ML |
|
1378 @cd Boogie; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL-Word HOL-Boogie |
|
1379 |
|
1380 |
|
1381 ## HOL-Boogie_Examples |
|
1382 |
|
1383 HOL-Boogie-Examples: HOL-Boogie $(LOG)/HOL-Boogie-Examples.gz |
|
1384 |
|
1385 $(LOG)/HOL-Boogie-Examples.gz: $(OUT)/HOL-Boogie \ |
|
1386 Boogie/Examples/ROOT.ML Boogie/Examples/Boogie_Max.thy \ |
|
1387 Boogie/Examples/Boogie_Max.b2i Boogie/Examples/Boogie_Dijkstra.thy \ |
|
1388 Boogie/Examples/VCC_Max.thy Boogie/Examples/Boogie_Dijkstra.b2i \ |
|
1389 Boogie/Examples/VCC_Max.b2i Boogie/Examples/Boogie_Max.certs \ |
|
1390 Boogie/Examples/Boogie_Dijkstra.certs Boogie/Examples/VCC_Max.certs |
|
1391 @cd Boogie; $(ISABELLE_TOOL) usedir $(OUT)/HOL-Boogie Examples |
|
1392 |
|
1393 |
|
1394 ## HOL-SPARK |
|
1395 |
|
1396 HOL-SPARK: HOL-Word $(OUT)/HOL-SPARK |
|
1397 |
|
1398 $(OUT)/HOL-SPARK: $(OUT)/HOL-Word SPARK/ROOT.ML \ |
|
1399 SPARK/SPARK.thy SPARK/SPARK_Setup.thy \ |
|
1400 SPARK/Tools/fdl_lexer.ML SPARK/Tools/fdl_parser.ML \ |
|
1401 SPARK/Tools/spark_commands.ML SPARK/Tools/spark_vcs.ML |
|
1402 @cd SPARK; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL-Word HOL-SPARK |
|
1403 |
|
1404 |
|
1405 ## HOL-SPARK-Examples |
|
1406 |
|
1407 HOL-SPARK-Examples: HOL-SPARK $(LOG)/HOL-SPARK-Examples.gz |
|
1408 |
|
1409 $(LOG)/HOL-SPARK-Examples.gz: $(OUT)/HOL-SPARK \ |
|
1410 SPARK/Examples/ROOT.ML \ |
|
1411 SPARK/Examples/Gcd/Greatest_Common_Divisor.thy \ |
|
1412 SPARK/Examples/Gcd/greatest_common_divisor/g_c_d.fdl \ |
|
1413 SPARK/Examples/Gcd/greatest_common_divisor/g_c_d.rls \ |
|
1414 SPARK/Examples/Gcd/greatest_common_divisor/g_c_d.siv \ |
|
1415 SPARK/Examples/Liseq/Longest_Increasing_Subsequence.thy \ |
|
1416 SPARK/Examples/Liseq/liseq/liseq_length.fdl \ |
|
1417 SPARK/Examples/Liseq/liseq/liseq_length.rls \ |
|
1418 SPARK/Examples/Liseq/liseq/liseq_length.siv \ |
|
1419 SPARK/Examples/RIPEMD-160/F.thy SPARK/Examples/RIPEMD-160/Hash.thy \ |
|
1420 SPARK/Examples/RIPEMD-160/K_L.thy SPARK/Examples/RIPEMD-160/K_R.thy \ |
|
1421 SPARK/Examples/RIPEMD-160/R_L.thy \ |
|
1422 SPARK/Examples/RIPEMD-160/RMD_Lemmas.thy \ |
|
1423 SPARK/Examples/RIPEMD-160/RMD_Specification.thy \ |
|
1424 SPARK/Examples/RIPEMD-160/RMD.thy SPARK/Examples/RIPEMD-160/Round.thy \ |
|
1425 SPARK/Examples/RIPEMD-160/R_R.thy SPARK/Examples/RIPEMD-160/S_L.thy \ |
|
1426 SPARK/Examples/RIPEMD-160/S_R.thy \ |
|
1427 SPARK/Examples/RIPEMD-160/rmd/f.fdl \ |
|
1428 SPARK/Examples/RIPEMD-160/rmd/f.rls \ |
|
1429 SPARK/Examples/RIPEMD-160/rmd/f.siv \ |
|
1430 SPARK/Examples/RIPEMD-160/rmd/hash.fdl \ |
|
1431 SPARK/Examples/RIPEMD-160/rmd/hash.rls \ |
|
1432 SPARK/Examples/RIPEMD-160/rmd/hash.siv \ |
|
1433 SPARK/Examples/RIPEMD-160/rmd/k_l.fdl \ |
|
1434 SPARK/Examples/RIPEMD-160/rmd/k_l.rls \ |
|
1435 SPARK/Examples/RIPEMD-160/rmd/k_l.siv \ |
|
1436 SPARK/Examples/RIPEMD-160/rmd/k_r.fdl \ |
|
1437 SPARK/Examples/RIPEMD-160/rmd/k_r.rls \ |
|
1438 SPARK/Examples/RIPEMD-160/rmd/k_r.siv \ |
|
1439 SPARK/Examples/RIPEMD-160/rmd/r_l.fdl \ |
|
1440 SPARK/Examples/RIPEMD-160/rmd/r_l.rls \ |
|
1441 SPARK/Examples/RIPEMD-160/rmd/r_l.siv \ |
|
1442 SPARK/Examples/RIPEMD-160/rmd/round.fdl \ |
|
1443 SPARK/Examples/RIPEMD-160/rmd/round.rls \ |
|
1444 SPARK/Examples/RIPEMD-160/rmd/round.siv \ |
|
1445 SPARK/Examples/RIPEMD-160/rmd/r_r.fdl \ |
|
1446 SPARK/Examples/RIPEMD-160/rmd/r_r.rls \ |
|
1447 SPARK/Examples/RIPEMD-160/rmd/r_r.siv \ |
|
1448 SPARK/Examples/RIPEMD-160/rmd/s_l.fdl \ |
|
1449 SPARK/Examples/RIPEMD-160/rmd/s_l.rls \ |
|
1450 SPARK/Examples/RIPEMD-160/rmd/s_l.siv \ |
|
1451 SPARK/Examples/RIPEMD-160/rmd/s_r.fdl \ |
|
1452 SPARK/Examples/RIPEMD-160/rmd/s_r.rls \ |
|
1453 SPARK/Examples/RIPEMD-160/rmd/s_r.siv |
|
1454 @cd SPARK; $(ISABELLE_TOOL) usedir $(OUT)/HOL-SPARK Examples |
|
1455 |
|
1456 |
|
1457 ## HOL-SPARK-Manual |
|
1458 |
|
1459 HOL-SPARK-Manual: HOL-SPARK $(LOG)/HOL-SPARK-Manual.gz |
|
1460 |
|
1461 $(LOG)/HOL-SPARK-Manual.gz: $(OUT)/HOL-SPARK \ |
|
1462 SPARK/Manual/ROOT.ML \ |
|
1463 SPARK/Manual/Complex_Types.thy \ |
|
1464 SPARK/Manual/Example_Verification.thy \ |
|
1465 SPARK/Manual/Proc1.thy \ |
|
1466 SPARK/Manual/Proc2.thy \ |
|
1467 SPARK/Manual/Reference.thy \ |
|
1468 SPARK/Manual/Simple_Greatest_Common_Divisor.thy \ |
|
1469 SPARK/Manual/VC_Principles.thy \ |
|
1470 SPARK/Manual/complex_types_app/initialize.fdl \ |
|
1471 SPARK/Manual/complex_types_app/initialize.rls \ |
|
1472 SPARK/Manual/complex_types_app/initialize.siv \ |
|
1473 SPARK/Manual/loop_invariant/proc1.fdl \ |
|
1474 SPARK/Manual/loop_invariant/proc1.rls \ |
|
1475 SPARK/Manual/loop_invariant/proc1.siv \ |
|
1476 SPARK/Manual/loop_invariant/proc2.fdl \ |
|
1477 SPARK/Manual/loop_invariant/proc2.rls \ |
|
1478 SPARK/Manual/loop_invariant/proc2.siv \ |
|
1479 SPARK/Manual/simple_greatest_common_divisor/g_c_d.fdl \ |
|
1480 SPARK/Manual/simple_greatest_common_divisor/g_c_d.rls \ |
|
1481 SPARK/Manual/simple_greatest_common_divisor/g_c_d.siv \ |
|
1482 SPARK/Manual/document/complex_types.ads \ |
|
1483 SPARK/Manual/document/complex_types_app.adb \ |
|
1484 SPARK/Manual/document/complex_types_app.ads \ |
|
1485 SPARK/Manual/document/loop_invariant.adb \ |
|
1486 SPARK/Manual/document/loop_invariant.ads \ |
|
1487 SPARK/Manual/document/Simple_Gcd.adb \ |
|
1488 SPARK/Manual/document/Simple_Gcd.ads \ |
|
1489 SPARK/Manual/document/intro.tex \ |
|
1490 SPARK/Manual/document/root.tex \ |
|
1491 SPARK/Manual/document/root.bib \ |
|
1492 SPARK/Examples/Gcd/Greatest_Common_Divisor.thy \ |
|
1493 SPARK/Examples/Gcd/greatest_common_divisor/g_c_d.fdl \ |
|
1494 SPARK/Examples/Gcd/greatest_common_divisor/g_c_d.rls \ |
|
1495 SPARK/Examples/Gcd/greatest_common_divisor/g_c_d.siv |
|
1496 @cd SPARK; $(ISABELLE_TOOL) usedir $(OUT)/HOL-SPARK Manual |
|
1497 |
|
1498 |
|
1499 ## HOL-Mutabelle |
|
1500 |
|
1501 HOL-Mutabelle: HOL $(LOG)/HOL-Mutabelle.gz |
|
1502 |
|
1503 $(LOG)/HOL-Mutabelle.gz: $(OUT)/HOL Mutabelle/MutabelleExtra.thy \ |
|
1504 Mutabelle/ROOT.ML Mutabelle/mutabelle.ML \ |
|
1505 Mutabelle/mutabelle_extra.ML |
|
1506 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Mutabelle |
|
1507 |
|
1508 ## HOL-Quickcheck_Examples |
|
1509 |
|
1510 HOL-Quickcheck_Examples: HOL $(LOG)/HOL-Quickcheck_Examples.gz |
|
1511 |
|
1512 $(LOG)/HOL-Quickcheck_Examples.gz: $(OUT)/HOL \ |
|
1513 Quickcheck_Examples/ROOT.ML \ |
|
1514 Quickcheck_Examples/Completeness.thy \ |
|
1515 Quickcheck_Examples/Hotel_Example.thy \ |
|
1516 Quickcheck_Examples/Quickcheck_Examples.thy \ |
|
1517 Quickcheck_Examples/Quickcheck_Interfaces.thy \ |
|
1518 Quickcheck_Examples/Quickcheck_Lattice_Examples.thy \ |
|
1519 Quickcheck_Examples/Quickcheck_Narrowing_Examples.thy |
|
1520 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Quickcheck_Examples |
|
1521 |
|
1522 ## HOL-Quotient_Examples |
|
1523 |
|
1524 HOL-Quotient_Examples: HOL $(LOG)/HOL-Quotient_Examples.gz |
|
1525 |
|
1526 $(LOG)/HOL-Quotient_Examples.gz: $(OUT)/HOL \ |
|
1527 Quotient_Examples/DList.thy \ |
|
1528 Quotient_Examples/FSet.thy \ |
|
1529 Quotient_Examples/Quotient_Int.thy Quotient_Examples/Quotient_Message.thy \ |
|
1530 Quotient_Examples/Lift_FSet.thy \ |
|
1531 Quotient_Examples/Lift_Set.thy \ |
|
1532 Quotient_Examples/Lift_Fun.thy Quotient_Examples/Lift_DList.thy |
|
1533 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Quotient_Examples |
|
1534 |
|
1535 |
|
1536 ## HOL-Predicate_Compile_Examples |
|
1537 |
|
1538 HOL-Predicate_Compile_Examples: HOL $(LOG)/HOL-Predicate_Compile_Examples.gz |
|
1539 |
|
1540 $(LOG)/HOL-Predicate_Compile_Examples.gz: $(OUT)/HOL \ |
|
1541 Predicate_Compile_Examples/ROOT.ML \ |
|
1542 Predicate_Compile_Examples/Predicate_Compile_Tests.thy \ |
|
1543 Predicate_Compile_Examples/Predicate_Compile_Quickcheck_Examples.thy \ |
|
1544 Predicate_Compile_Examples/Code_Prolog_Examples.thy \ |
|
1545 Predicate_Compile_Examples/Examples.thy \ |
|
1546 Predicate_Compile_Examples/Context_Free_Grammar_Example.thy \ |
|
1547 Predicate_Compile_Examples/Hotel_Example.thy \ |
|
1548 Predicate_Compile_Examples/Hotel_Example_Prolog.thy \ |
|
1549 Predicate_Compile_Examples/Hotel_Example_Small_Generator.thy \ |
|
1550 Predicate_Compile_Examples/IMP_1.thy \ |
|
1551 Predicate_Compile_Examples/IMP_2.thy \ |
|
1552 Predicate_Compile_Examples/IMP_3.thy \ |
|
1553 Predicate_Compile_Examples/IMP_4.thy \ |
|
1554 Predicate_Compile_Examples/Lambda_Example.thy \ |
|
1555 Predicate_Compile_Examples/List_Examples.thy \ |
|
1556 Predicate_Compile_Examples/Reg_Exp_Example.thy |
|
1557 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Predicate_Compile_Examples |
|
1558 |
|
1559 |
|
1560 ## HOLCF |
|
1561 |
|
1562 HOLCF: HOL $(OUT)/HOLCF |
|
1563 |
|
1564 $(OUT)/HOLCF: $(OUT)/HOL \ |
|
1565 HOLCF/ROOT.ML \ |
|
1566 HOLCF/Adm.thy \ |
|
1567 HOLCF/Algebraic.thy \ |
|
1568 HOLCF/Bifinite.thy \ |
|
1569 HOLCF/Cfun.thy \ |
|
1570 HOLCF/Compact_Basis.thy \ |
|
1571 HOLCF/Completion.thy \ |
|
1572 HOLCF/Cont.thy \ |
|
1573 HOLCF/ConvexPD.thy \ |
|
1574 HOLCF/Cpodef.thy \ |
|
1575 HOLCF/Cprod.thy \ |
|
1576 HOLCF/Discrete.thy \ |
|
1577 HOLCF/Deflation.thy \ |
|
1578 HOLCF/Domain.thy \ |
|
1579 HOLCF/Domain_Aux.thy \ |
|
1580 HOLCF/Fixrec.thy \ |
|
1581 HOLCF/Fix.thy \ |
|
1582 HOLCF/Fun_Cpo.thy \ |
|
1583 HOLCF/HOLCF.thy \ |
|
1584 HOLCF/Lift.thy \ |
|
1585 HOLCF/LowerPD.thy \ |
|
1586 HOLCF/Map_Functions.thy \ |
|
1587 HOLCF/One.thy \ |
|
1588 HOLCF/Pcpo.thy \ |
|
1589 HOLCF/Plain_HOLCF.thy \ |
|
1590 HOLCF/Porder.thy \ |
|
1591 HOLCF/Powerdomains.thy \ |
|
1592 HOLCF/Product_Cpo.thy \ |
|
1593 HOLCF/Representable.thy \ |
|
1594 HOLCF/Sfun.thy \ |
|
1595 HOLCF/Sprod.thy \ |
|
1596 HOLCF/Ssum.thy \ |
|
1597 HOLCF/Tr.thy \ |
|
1598 HOLCF/Universal.thy \ |
|
1599 HOLCF/UpperPD.thy \ |
|
1600 HOLCF/Up.thy \ |
|
1601 HOLCF/Tools/cont_consts.ML \ |
|
1602 HOLCF/Tools/cont_proc.ML \ |
|
1603 HOLCF/Tools/holcf_library.ML \ |
|
1604 HOLCF/Tools/Domain/domain.ML \ |
|
1605 HOLCF/Tools/Domain/domain_axioms.ML \ |
|
1606 HOLCF/Tools/Domain/domain_constructors.ML \ |
|
1607 HOLCF/Tools/Domain/domain_induction.ML \ |
|
1608 HOLCF/Tools/Domain/domain_isomorphism.ML \ |
|
1609 HOLCF/Tools/Domain/domain_take_proofs.ML \ |
|
1610 HOLCF/Tools/cpodef.ML \ |
|
1611 HOLCF/Tools/domaindef.ML \ |
|
1612 HOLCF/Tools/fixrec.ML \ |
|
1613 HOLCF/document/root.tex |
|
1614 @cd HOLCF; $(ISABELLE_TOOL) usedir -b -g true $(OUT)/HOL HOLCF |
|
1615 |
|
1616 |
|
1617 ## HOLCF-Tutorial |
|
1618 |
|
1619 HOLCF-Tutorial: HOLCF $(LOG)/HOLCF-Tutorial.gz |
|
1620 |
|
1621 $(LOG)/HOLCF-Tutorial.gz: $(OUT)/HOLCF \ |
|
1622 HOLCF/Tutorial/Domain_ex.thy \ |
|
1623 HOLCF/Tutorial/Fixrec_ex.thy \ |
|
1624 HOLCF/Tutorial/New_Domain.thy \ |
|
1625 HOLCF/Tutorial/document/root.tex \ |
|
1626 HOLCF/Tutorial/ROOT.ML |
|
1627 @cd HOLCF; $(ISABELLE_TOOL) usedir $(OUT)/HOLCF Tutorial |
|
1628 |
|
1629 |
|
1630 ## HOLCF-Library |
|
1631 |
|
1632 HOLCF-Library: HOLCF $(LOG)/HOLCF-Library.gz |
|
1633 |
|
1634 $(LOG)/HOLCF-Library.gz: $(OUT)/HOLCF \ |
|
1635 Library/Extended_Nat.thy \ |
|
1636 HOLCF/Library/Defl_Bifinite.thy \ |
|
1637 HOLCF/Library/Bool_Discrete.thy \ |
|
1638 HOLCF/Library/Char_Discrete.thy \ |
|
1639 HOLCF/Library/HOL_Cpo.thy \ |
|
1640 HOLCF/Library/Int_Discrete.thy \ |
|
1641 HOLCF/Library/List_Cpo.thy \ |
|
1642 HOLCF/Library/List_Predomain.thy \ |
|
1643 HOLCF/Library/Nat_Discrete.thy \ |
|
1644 HOLCF/Library/Option_Cpo.thy \ |
|
1645 HOLCF/Library/Stream.thy \ |
|
1646 HOLCF/Library/Sum_Cpo.thy \ |
|
1647 HOLCF/Library/HOLCF_Library.thy \ |
|
1648 HOLCF/Library/ROOT.ML |
|
1649 @cd HOLCF; $(ISABELLE_TOOL) usedir $(OUT)/HOLCF Library |
|
1650 |
|
1651 |
|
1652 ## HOLCF-IMP |
|
1653 |
|
1654 HOLCF-IMP: HOLCF $(LOG)/HOLCF-IMP.gz |
|
1655 |
|
1656 $(LOG)/HOLCF-IMP.gz: $(OUT)/HOLCF \ |
|
1657 HOLCF/IMP/HoareEx.thy \ |
|
1658 HOLCF/IMP/Denotational.thy \ |
|
1659 HOLCF/IMP/ROOT.ML \ |
|
1660 HOLCF/IMP/document/root.tex |
|
1661 @cd HOLCF; $(ISABELLE_TOOL) usedir $(OUT)/HOLCF IMP |
|
1662 |
|
1663 |
|
1664 ## HOLCF-ex |
|
1665 |
|
1666 HOLCF-ex: HOLCF $(LOG)/HOLCF-ex.gz |
|
1667 |
|
1668 $(LOG)/HOLCF-ex.gz: $(OUT)/HOLCF \ |
|
1669 HOLCF/ex/Concurrency_Monad.thy \ |
|
1670 HOLCF/ex/Dagstuhl.thy \ |
|
1671 HOLCF/ex/Dnat.thy \ |
|
1672 HOLCF/ex/Domain_Proofs.thy \ |
|
1673 HOLCF/ex/Fix2.thy \ |
|
1674 HOLCF/ex/Focus_ex.thy \ |
|
1675 HOLCF/ex/Hoare.thy \ |
|
1676 HOLCF/ex/Letrec.thy \ |
|
1677 HOLCF/ex/Loop.thy \ |
|
1678 HOLCF/ex/Pattern_Match.thy \ |
|
1679 HOLCF/ex/Powerdomain_ex.thy \ |
|
1680 HOLCF/ex/ROOT.ML |
|
1681 @cd HOLCF; $(ISABELLE_TOOL) usedir $(OUT)/HOLCF ex |
|
1682 |
|
1683 |
|
1684 ## HOLCF-FOCUS |
|
1685 |
|
1686 HOLCF-FOCUS: HOLCF $(LOG)/HOLCF-FOCUS.gz |
|
1687 |
|
1688 $(LOG)/HOLCF-FOCUS.gz: $(OUT)/HOLCF HOLCF/FOCUS/ROOT.ML \ |
|
1689 Library/Extended_Nat.thy \ |
|
1690 HOLCF/Library/Stream.thy \ |
|
1691 HOLCF/FOCUS/Fstreams.thy \ |
|
1692 HOLCF/FOCUS/Fstream.thy \ |
|
1693 HOLCF/FOCUS/FOCUS.thy \ |
|
1694 HOLCF/FOCUS/Stream_adm.thy \ |
|
1695 HOLCF/FOCUS/Buffer.thy \ |
|
1696 HOLCF/FOCUS/Buffer_adm.thy \ |
|
1697 Library/Continuity.thy |
|
1698 @cd HOLCF; $(ISABELLE_TOOL) usedir $(OUT)/HOLCF FOCUS |
|
1699 |
|
1700 |
|
1701 ## IOA |
|
1702 |
|
1703 IOA: HOLCF $(OUT)/IOA |
|
1704 |
|
1705 $(OUT)/IOA: $(OUT)/HOLCF \ |
|
1706 HOLCF/IOA/ROOT.ML \ |
|
1707 HOLCF/IOA/meta_theory/Traces.thy \ |
|
1708 HOLCF/IOA/meta_theory/Asig.thy \ |
|
1709 HOLCF/IOA/meta_theory/CompoScheds.thy \ |
|
1710 HOLCF/IOA/meta_theory/CompoTraces.thy \ |
|
1711 HOLCF/IOA/meta_theory/Seq.thy \ |
|
1712 HOLCF/IOA/meta_theory/RefCorrectness.thy \ |
|
1713 HOLCF/IOA/meta_theory/Automata.thy \ |
|
1714 HOLCF/IOA/meta_theory/ShortExecutions.thy \ |
|
1715 HOLCF/IOA/meta_theory/IOA.thy \ |
|
1716 HOLCF/IOA/meta_theory/Sequence.thy \ |
|
1717 HOLCF/IOA/meta_theory/CompoExecs.thy \ |
|
1718 HOLCF/IOA/meta_theory/RefMappings.thy \ |
|
1719 HOLCF/IOA/meta_theory/Compositionality.thy \ |
|
1720 HOLCF/IOA/meta_theory/TL.thy \ |
|
1721 HOLCF/IOA/meta_theory/TLS.thy \ |
|
1722 HOLCF/IOA/meta_theory/LiveIOA.thy \ |
|
1723 HOLCF/IOA/meta_theory/Pred.thy \ |
|
1724 HOLCF/IOA/meta_theory/Abstraction.thy \ |
|
1725 HOLCF/IOA/meta_theory/Simulations.thy \ |
|
1726 HOLCF/IOA/meta_theory/SimCorrectness.thy |
|
1727 @cd HOLCF/IOA; $(ISABELLE_TOOL) usedir -b $(OUT)/HOLCF IOA |
|
1728 |
|
1729 |
|
1730 ## IOA-ABP |
|
1731 |
|
1732 IOA-ABP: IOA $(LOG)/IOA-ABP.gz |
|
1733 |
|
1734 $(LOG)/IOA-ABP.gz: $(OUT)/IOA \ |
|
1735 HOLCF/IOA/ABP/Abschannel.thy \ |
|
1736 HOLCF/IOA/ABP/Abschannel_finite.thy \ |
|
1737 HOLCF/IOA/ABP/Action.thy \ |
|
1738 HOLCF/IOA/ABP/Check.ML \ |
|
1739 HOLCF/IOA/ABP/Correctness.thy \ |
|
1740 HOLCF/IOA/ABP/Env.thy \ |
|
1741 HOLCF/IOA/ABP/Impl.thy \ |
|
1742 HOLCF/IOA/ABP/Impl_finite.thy \ |
|
1743 HOLCF/IOA/ABP/Lemmas.thy \ |
|
1744 HOLCF/IOA/ABP/Packet.thy \ |
|
1745 HOLCF/IOA/ABP/ROOT.ML \ |
|
1746 HOLCF/IOA/ABP/Receiver.thy \ |
|
1747 HOLCF/IOA/ABP/Sender.thy \ |
|
1748 HOLCF/IOA/ABP/Spec.thy |
|
1749 @cd HOLCF/IOA; $(ISABELLE_TOOL) usedir $(OUT)/IOA ABP |
|
1750 |
|
1751 |
|
1752 ## IOA-NTP |
|
1753 |
|
1754 IOA-NTP: IOA $(LOG)/IOA-NTP.gz |
|
1755 |
|
1756 $(LOG)/IOA-NTP.gz: $(OUT)/IOA \ |
|
1757 HOLCF/IOA/NTP/Abschannel.thy \ |
|
1758 HOLCF/IOA/NTP/Action.thy \ |
|
1759 HOLCF/IOA/NTP/Correctness.thy \ |
|
1760 HOLCF/IOA/NTP/Impl.thy \ |
|
1761 HOLCF/IOA/NTP/Lemmas.thy \ |
|
1762 HOLCF/IOA/NTP/Multiset.thy \ |
|
1763 HOLCF/IOA/NTP/Packet.thy \ |
|
1764 HOLCF/IOA/NTP/ROOT.ML \ |
|
1765 HOLCF/IOA/NTP/Receiver.thy \ |
|
1766 HOLCF/IOA/NTP/Sender.thy \ |
|
1767 HOLCF/IOA/NTP/Spec.thy |
|
1768 @cd HOLCF/IOA; $(ISABELLE_TOOL) usedir $(OUT)/IOA NTP |
|
1769 |
|
1770 |
|
1771 ## IOA-Storage |
|
1772 |
|
1773 IOA-Storage: IOA $(LOG)/IOA-Storage.gz |
|
1774 |
|
1775 $(LOG)/IOA-Storage.gz: $(OUT)/IOA \ |
|
1776 HOLCF/IOA/Storage/Action.thy \ |
|
1777 HOLCF/IOA/Storage/Correctness.thy \ |
|
1778 HOLCF/IOA/Storage/Impl.thy \ |
|
1779 HOLCF/IOA/Storage/ROOT.ML \ |
|
1780 HOLCF/IOA/Storage/Spec.thy |
|
1781 @cd HOLCF/IOA; $(ISABELLE_TOOL) usedir $(OUT)/IOA Storage |
|
1782 |
|
1783 |
|
1784 ## IOA-ex |
|
1785 |
|
1786 IOA-ex: IOA $(LOG)/IOA-ex.gz |
|
1787 |
|
1788 $(LOG)/IOA-ex.gz: $(OUT)/IOA \ |
|
1789 HOLCF/IOA/ex/ROOT.ML \ |
|
1790 HOLCF/IOA/ex/TrivEx.thy \ |
|
1791 HOLCF/IOA/ex/TrivEx2.thy |
|
1792 @cd HOLCF/IOA; $(ISABELLE_TOOL) usedir $(OUT)/IOA ex |
|
1793 |
|
1794 |
|
1795 |
|
1796 ## HOL-Datatype_Benchmark |
|
1797 |
|
1798 HOL-Datatype_Benchmark: HOL $(LOG)/HOL-Datatype_Benchmark.gz |
|
1799 |
|
1800 $(LOG)/HOL-Datatype_Benchmark.gz: $(OUT)/HOL \ |
|
1801 Datatype_Benchmark/ROOT.ML Datatype_Benchmark/Brackin.thy \ |
|
1802 Datatype_Benchmark/Instructions.thy Datatype_Benchmark/SML.thy \ |
|
1803 Datatype_Benchmark/Verilog.thy |
|
1804 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Datatype_Benchmark |
|
1805 |
|
1806 |
|
1807 ## HOL-Record_Benchmark |
|
1808 |
|
1809 HOL-Record_Benchmark: HOL $(LOG)/HOL-Record_Benchmark.gz |
|
1810 |
|
1811 $(LOG)/HOL-Record_Benchmark.gz: $(OUT)/HOL Record_Benchmark/ROOT.ML \ |
|
1812 Record_Benchmark/Record_Benchmark.thy |
|
1813 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Record_Benchmark |
|
1814 |
|
1815 |
|
1816 ## HOL-Quickcheck_Benchmark |
|
1817 |
|
1818 HOL-Quickcheck_Benchmark: HOL $(LOG)/HOL-Quickcheck_Benchmark.gz |
|
1819 |
|
1820 $(LOG)/HOL-Quickcheck_Benchmark.gz: $(OUT)/HOL \ |
|
1821 Quickcheck_Benchmark/ROOT.ML \ |
|
1822 Quickcheck_Benchmark/Needham_Schroeder_Base.thy \ |
|
1823 Quickcheck_Benchmark/Needham_Schroeder_No_Attacker_Example.thy \ |
|
1824 Quickcheck_Benchmark/Needham_Schroeder_Guided_Attacker_Example.thy \ |
|
1825 Quickcheck_Benchmark/Needham_Schroeder_Unguided_Attacker_Example.thy \ |
|
1826 Quickcheck_Benchmark/Find_Unused_Assms_Examples.thy |
|
1827 @$(ISABELLE_TOOL) usedir $(OUT)/HOL Quickcheck_Benchmark |
|
1828 |
|
1829 |
|
1830 ## clean |
|
1831 |
|
1832 clean: |
|
1833 @rm -f $(LOG)/HOL-Algebra.gz $(LOG)/HOL-Auth.gz \ |
|
1834 $(LOG)/HOL-Bali.gz $(LOG)/HOL-Base.gz \ |
|
1835 $(LOG)/HOL-Boogie-Examples.gz $(LOG)/HOL-Boogie.gz \ |
|
1836 $(LOG)/HOL-Decision_Procs.gz $(LOG)/HOL-HOL_Light.gz \ |
|
1837 $(LOG)/HOL-Hahn_Banach.gz $(LOG)/HOL-Hoare.gz \ |
|
1838 $(LOG)/HOL-Hoare_Parallel.gz $(LOG)/HOL-IMP.gz \ |
|
1839 $(LOG)/HOL-IMPP.gz $(LOG)/HOL-IOA.gz \ |
|
1840 $(LOG)/HOL-Imperative_HOL.gz $(LOG)/HOL-Import.gz \ |
|
1841 $(LOG)/HOL-Induct.gz $(LOG)/HOL-Isar_Examples.gz \ |
|
1842 $(LOG)/HOL-Lattice $(LOG)/HOL-Lattice.gz \ |
|
1843 $(LOG)/HOL-Lex.gz $(LOG)/HOL-Library.gz \ |
|
1844 $(LOG)/HOL-Library-Codegenerator_Test.gz \ |
|
1845 $(LOG)/HOL-Main.gz $(LOG)/HOL-Matrix_LP.gz \ |
|
1846 $(LOG)/HOL-Metis_Examples.gz $(LOG)/HOL-MicroJava.gz \ |
|
1847 $(LOG)/HOL-Mirabelle.gz \ |
|
1848 $(LOG)/HOL-Multivariate_Analysis.gz \ |
|
1849 $(LOG)/HOL-Mutabelle.gz $(LOG)/HOL-NSA-Examples.gz \ |
|
1850 $(LOG)/HOL-NSA.gz $(LOG)/HOL-NanoJava.gz \ |
|
1851 $(LOG)/HOL-Nitpick_Examples.gz \ |
|
1852 $(LOG)/HOL-Nominal-Examples.gz $(LOG)/HOL-Nominal.gz \ |
|
1853 $(LOG)/HOL-Number_Theory.gz \ |
|
1854 $(LOG)/HOL-Old_Number_Theory.gz $(LOG)/HOL-Plain.gz \ |
|
1855 $(LOG)/HOL-Predicate_Compile_Examples.gz \ |
|
1856 $(LOG)/HOL-Probability.gz $(LOG)/HOL-Prolog.gz \ |
|
1857 $(LOG)/HOL-Proofs.gz $(LOG)/HOL-Proofs-ex.gz \ |
|
1858 $(LOG)/HOL-Proofs-Extraction.gz \ |
|
1859 $(LOG)/HOL-Proofs-Lambda.gz \ |
|
1860 $(LOG)/HOL-Quickcheck_Examples.gz \ |
|
1861 $(LOG)/HOL-Quotient_Examples.gz \ |
|
1862 $(LOG)/HOL-SET_Protocol.gz \ |
|
1863 $(LOG)/HOL-Word-SMT_Examples.gz $(LOG)/HOL-SPARK.gz \ |
|
1864 $(LOG)/HOL-SPARK-Examples.gz \ |
|
1865 $(LOG)/HOL-SPARK-Manual.gz $(LOG)/HOL-Statespace.gz \ |
|
1866 $(LOG)/HOL-TPTP.gz $(LOG)/HOL-UNITY.gz \ |
|
1867 $(LOG)/HOL-Unix.gz $(LOG)/HOL-Word-Examples.gz \ |
|
1868 $(LOG)/HOL-Word.gz $(LOG)/HOL-ZF.gz $(LOG)/HOL-ex.gz \ |
|
1869 $(LOG)/HOL.gz $(LOG)/TLA-Buffer.gz $(LOG)/TLA-Inc.gz \ |
|
1870 $(LOG)/TLA-Memory.gz $(LOG)/TLA.gz $(OUT)/HOL \ |
|
1871 $(OUT)/HOL-Algebra $(OUT)/HOL-Base $(OUT)/HOL-Boogie \ |
|
1872 $(OUT)/HOL-HOL_Light $(OUT)/HOL-IMP $(OUT)/HOL-Library \ |
|
1873 $(OUT)/HOL-Main $(OUT)/HOL-Multivariate_Analysis \ |
|
1874 $(OUT)/HOL-NSA $(OUT)/HOL-Nominal $(OUT)/HOL-Plain \ |
|
1875 $(OUT)/HOL-Probability $(OUT)/HOL-Proofs \ |
|
1876 $(OUT)/HOL-SPARK $(OUT)/HOL-Word $(OUT)/TLA \ |
|
1877 $(OUT)/HOLCF $(LOG)/HOLCF.gz $(LOG)/HOLCF-IMP.gz \ |
|
1878 $(LOG)/HOLCF-ex.gz $(LOG)/HOLCF-FOCUS.gz $(OUT)/IOA \ |
|
1879 $(LOG)/IOA.gz $(LOG)/IOA-ABP.gz $(LOG)/IOA-NTP.gz \ |
|
1880 $(LOG)/IOA-Storage.gz $(LOG)/HOLCF-Library.gz \ |
|
1881 $(LOG)/IOA-ex.gz $(LOG)/HOLCF-Tutorial.gz \ |
|
1882 $(LOG)/HOL-Datatype_Benchmark.gz \ |
|
1883 $(LOG)/HOL-Record_Benchmark.gz |
|