author | blanchet |
Mon, 21 May 2012 10:39:31 +0200 | |
changeset 47944 | e6b51fab96f7 |
parent 47509 | 6f215c2ebd72 |
child 48891 | c0eafbd55de3 |
permissions | -rw-r--r-- |
46844 | 1 |
(* Title: HOL/TPTP/TPTP_Parser.thy |
2 |
Author: Nik Sultana, Cambridge University Computer Laboratory |
|
3 |
||
47509
6f215c2ebd72
split TPTP_Parser thy -- parser can rely on smaller image, whereas TPTP_Interpret requires HOL;
sultana
parents:
47411
diff
changeset
|
4 |
Parser for TPTP formulas |
46844 | 5 |
*) |
6 |
||
7 |
theory TPTP_Parser |
|
47509
6f215c2ebd72
split TPTP_Parser thy -- parser can rely on smaller image, whereas TPTP_Interpret requires HOL;
sultana
parents:
47411
diff
changeset
|
8 |
imports Pure |
46844 | 9 |
uses |
10 |
"TPTP_Parser/ml_yacc_lib.ML" (*generated from ML-Yacc's lib*) |
|
11 |
||
12 |
"TPTP_Parser/tptp_syntax.ML" |
|
13 |
"TPTP_Parser/tptp_lexyacc.ML" (*generated from tptp.lex and tptp.yacc*) |
|
14 |
"TPTP_Parser/tptp_parser.ML" |
|
15 |
"TPTP_Parser/tptp_problem_name.ML" |
|
47411
7df9a4f320a5
moved non-interpret-specific code to different module
sultana
parents:
46951
diff
changeset
|
16 |
"TPTP_Parser/tptp_proof.ML" |
46844 | 17 |
|
18 |
begin |
|
19 |
||
20 |
text {*The TPTP parser was generated using ML-Yacc, and needs the |
|
21 |
ML-Yacc library to operate. This library is included with the parser, |
|
22 |
and we include the next section in accordance with ML-Yacc's terms of |
|
23 |
use.*} |
|
24 |
||
25 |
section "ML-YACC COPYRIGHT NOTICE, LICENSE AND DISCLAIMER." |
|
26 |
text {* |
|
27 |
Copyright 1989, 1990 by David R. Tarditi Jr. and Andrew W. Appel |
|
28 |
||
29 |
Permission to use, copy, modify, and distribute this software and its |
|
30 |
documentation for any purpose and without fee is hereby granted, |
|
31 |
provided that the above copyright notice appear in all copies and that |
|
32 |
both the copyright notice and this permission notice and warranty |
|
33 |
disclaimer appear in supporting documentation, and that the names of |
|
34 |
David R. Tarditi Jr. and Andrew W. Appel not be used in advertising or |
|
35 |
publicity pertaining to distribution of the software without specific, |
|
36 |
written prior permission. |
|
37 |
||
38 |
David R. Tarditi Jr. and Andrew W. Appel disclaim all warranties with |
|
39 |
regard to this software, including all implied warranties of |
|
40 |
merchantability and fitness. In no event shall David R. Tarditi |
|
41 |
Jr. and Andrew W. Appel be liable for any special, indirect or |
|
42 |
consequential damages or any damages whatsoever resulting from loss of |
|
43 |
use, data or profits, whether in an action of contract, negligence or |
|
44 |
other tortious action, arising out of or in connection with the use or |
|
45 |
performance of this software. |
|
46 |
*} |
|
47 |
||
48 |
end |