Fri, 24 Nov 2006 16:38:42 +0100 |
paulson |
Conversion of "equal" to "=" for TSTP format; big tidy-up
|
changeset |
files
|
Fri, 24 Nov 2006 13:44:51 +0100 |
krauss |
Lemma "fundef_default_value" uses predicate instead of set.
|
changeset |
files
|
Fri, 24 Nov 2006 13:43:44 +0100 |
krauss |
The function package declares the [code] attribute automatically again.
|
changeset |
files
|
Fri, 24 Nov 2006 13:39:22 +0100 |
krauss |
exported mk_base_funs for use by size-change tools
|
changeset |
files
|
Fri, 24 Nov 2006 13:24:30 +0100 |
paulson |
ATP linkup now generates "new TPTP" rather than "old TPTP"
|
changeset |
files
|
Thu, 23 Nov 2006 23:05:28 +0100 |
wenzelm |
more careful declaration of "inducts";
|
changeset |
files
|
Thu, 23 Nov 2006 22:38:32 +0100 |
wenzelm |
tuned;
|
changeset |
files
|
Thu, 23 Nov 2006 22:38:30 +0100 |
wenzelm |
prefer Proof.context over Context.generic;
|
changeset |
files
|
Thu, 23 Nov 2006 22:38:29 +0100 |
wenzelm |
prefer Proof.context over Context.generic;
|
changeset |
files
|
Thu, 23 Nov 2006 22:38:28 +0100 |
wenzelm |
tuned proofs;
|
changeset |
files
|
Thu, 23 Nov 2006 22:14:26 +0100 |
aspinall |
Accept URLs of form file:/home... also.
|
changeset |
files
|
Thu, 23 Nov 2006 20:34:21 +0100 |
wenzelm |
prefer antiquotations over LaTeX macros;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:42 +0100 |
wenzelm |
updated;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:41 +0100 |
wenzelm |
renamed Args.Name to Args.Text;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:39 +0100 |
wenzelm |
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:37 +0100 |
wenzelm |
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:36 +0100 |
wenzelm |
Morphism.thm_morphism;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:34 +0100 |
wenzelm |
renamed Name value to Text, which is *not* a name in terms of morphisms;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:33 +0100 |
wenzelm |
removed obsolete alphanum;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:32 +0100 |
wenzelm |
str_of_char: improved output of non-printables;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:29 +0100 |
wenzelm |
added head_name_of;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:28 +0100 |
wenzelm |
added name/var/typ/term/thm_morphism;
|
changeset |
files
|
Thu, 23 Nov 2006 20:33:25 +0100 |
wenzelm |
declarations: pass morphism (dummy);
|
changeset |
files
|
Thu, 23 Nov 2006 18:49:55 +0100 |
wenzelm |
added ISABELLE_IDENTIFIER;
|
changeset |
files
|
Thu, 23 Nov 2006 18:49:03 +0100 |
wenzelm |
ISABELLE_PATH/OUTPUT: append ISABELLE_IDENTIFIER if derived from ISABELLE_HOME_USER;
|
changeset |
files
|
Thu, 23 Nov 2006 17:52:48 +0100 |
urbanc |
fixed some typos
|
changeset |
files
|
Thu, 23 Nov 2006 14:11:49 +0100 |
urbanc |
tuned the proof of the strong induction principle
|
changeset |
files
|
Thu, 23 Nov 2006 13:32:19 +0100 |
webertj |
typo in comment fixed
|
changeset |
files
|
Thu, 23 Nov 2006 11:39:11 +0100 |
aspinall |
Add retractfile to supported pgip commands
|
changeset |
files
|
Thu, 23 Nov 2006 11:24:33 +0100 |
aspinall |
PGIP: add retractfile. Be stricter in file open/close protocol.
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:23 +0100 |
wenzelm |
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:19 +0100 |
wenzelm |
moved ML identifiers to structure ML_Syntax;
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:15 +0100 |
wenzelm |
added morph_ctxt, morph_witness;
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:11 +0100 |
wenzelm |
replaced map_values by morph_values;
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:07 +0100 |
wenzelm |
moved string_of_pair/list/option to structure ML_Syntax;
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:03 +0100 |
wenzelm |
moved ML syntax operations to structure ML_Syntax;
|
changeset |
files
|
Thu, 23 Nov 2006 00:52:01 +0100 |
wenzelm |
Basic ML syntax operations.
|
changeset |
files
|
Thu, 23 Nov 2006 00:51:57 +0100 |
wenzelm |
Abstract morphisms on formal entities.
|
changeset |
files
|
Thu, 23 Nov 2006 00:51:54 +0100 |
wenzelm |
added morphism.ML, General/ml_syntax.ML;
|
changeset |
files
|
Thu, 23 Nov 2006 00:51:51 +0100 |
wenzelm |
renamed string_of_pair/list/option to ML_Syntax.str_of_pair/list/option;
|
changeset |
files
|
Thu, 23 Nov 2006 00:51:47 +0100 |
wenzelm |
removed dead code;
|
changeset |
files
|
Thu, 23 Nov 2006 00:09:24 +0100 |
aspinall |
Add doccomment; rename litcomment -> doccomment
|
changeset |
files
|
Wed, 22 Nov 2006 20:51:00 +0100 |
wenzelm |
* settings: ML_IDENTIFIER includes the Isabelle version identifier;
|
changeset |
files
|
Wed, 22 Nov 2006 20:08:07 +0100 |
paulson |
Consolidation of code to "blacklist" unhelpful theorems, including record
|
changeset |
files
|
Wed, 22 Nov 2006 19:55:22 +0100 |
wenzelm |
ML_IDENTIFIER includes Isabelle version;
|
changeset |
files
|
Wed, 22 Nov 2006 19:53:24 +0100 |
wenzelm |
add ISABELLE_VERSION to ML_IDENTIFIER, unless this is repository or build;
|
changeset |
files
|
Wed, 22 Nov 2006 17:38:36 +0100 |
wenzelm |
consts: ProofContext.set_stmt true -- avoids naming of local thms;
|
changeset |
files
|
Wed, 22 Nov 2006 15:58:59 +0100 |
wenzelm |
init: enter inner statement mode, which prevents local notes from being named internally;
|
changeset |
files
|
Wed, 22 Nov 2006 15:58:15 +0100 |
wenzelm |
more careful declaration of "intros" as Pure.intro;
|
changeset |
files
|
Wed, 22 Nov 2006 12:01:59 +0100 |
aspinall |
Fix to local file URI syntax. Add first part of lexicalstructure command support.
|
changeset |
files
|
Wed, 22 Nov 2006 10:22:04 +0100 |
haftmann |
completed class parameter handling in axclass.ML
|
changeset |
files
|
Wed, 22 Nov 2006 10:21:17 +0100 |
haftmann |
added Isar syntax for adding parameters to axclasses
|
changeset |
files
|
Wed, 22 Nov 2006 10:20:22 +0100 |
haftmann |
forced name prefix for class operations
|
changeset |
files
|
Wed, 22 Nov 2006 10:20:20 +0100 |
haftmann |
example tuned
|
changeset |
files
|
Wed, 22 Nov 2006 10:20:19 +0100 |
haftmann |
no explicit check for theory Nat
|
changeset |
files
|
Wed, 22 Nov 2006 10:20:18 +0100 |
haftmann |
added code lemmas
|
changeset |
files
|