wenzelm [Thu, 03 Apr 2008 21:23:41 +0200] rev 26549
moved test_markup here;
wenzelm [Thu, 03 Apr 2008 21:23:39 +0200] rev 26548
further cleanup of XML signature;
wenzelm [Thu, 03 Apr 2008 21:23:38 +0200] rev 26547
tuned comments;
wenzelm [Thu, 03 Apr 2008 21:23:37 +0200] rev 26546
further cleanup of XML signature;
replaced plain_content by incremental add_content;
added stream output;
wenzelm [Thu, 03 Apr 2008 21:23:36 +0200] rev 26545
output: canonical argument order (as opposed to write);
wenzelm [Thu, 03 Apr 2008 18:42:42 +0200] rev 26544
XML.string_of;
wenzelm [Thu, 03 Apr 2008 18:42:41 +0200] rev 26543
moved output_markup to xml.ML;
added yxmlN mode name;
wenzelm [Thu, 03 Apr 2008 18:42:40 +0200] rev 26542
XML.output_markup;
wenzelm [Thu, 03 Apr 2008 18:42:39 +0200] rev 26541
XML.string_of, XML.parse;
wenzelm [Thu, 03 Apr 2008 18:42:38 +0200] rev 26540
replaced ETX/EOT by ENQ/ACK, which are less likely to be interpreted by tty etc.;
added output_markup, parse_element;
detect: check XY;
tuned comments;
tuned;
wenzelm [Thu, 03 Apr 2008 18:42:37 +0200] rev 26539
added output_markup (from Tools/isabelle_process.ML);
major cleanup of signature;
wenzelm [Thu, 03 Apr 2008 18:42:36 +0200] rev 26538
replaced ETX/EOT by ENQ/ACK, which are less likely to be interpreted by tty etc.;
wenzelm [Thu, 03 Apr 2008 18:42:34 +0200] rev 26537
tuned comments;
berghofe [Thu, 03 Apr 2008 18:13:50 +0200] rev 26536
Added skip_mono flag to inductive definition package.
berghofe [Thu, 03 Apr 2008 17:55:12 +0200] rev 26535
Added skip_mono flag to inductive definition package.
berghofe [Thu, 03 Apr 2008 17:54:19 +0200] rev 26534
Added skip_mono flag and inductive_flags type.
berghofe [Thu, 03 Apr 2008 17:52:51 +0200] rev 26533
Deleted code for axiomatic introduction of datatypes. Instead, the package
now uses SkipProof.prove rather than Goal.prove to do proofs.
berghofe [Thu, 03 Apr 2008 17:50:50 +0200] rev 26532
Removed QuickAndDirty constructor from simproc_dist datatype.
berghofe [Thu, 03 Apr 2008 17:49:39 +0200] rev 26531
- use SkipProof.prove_global instead of Goal.prove_global
- added skip_mono flag to inductive definition package
berghofe [Thu, 03 Apr 2008 17:43:01 +0200] rev 26530
Added prove_global.
krauss [Thu, 03 Apr 2008 16:34:52 +0200] rev 26529
Function package no longer overwrites theorems.
Some tuning.
wenzelm [Thu, 03 Apr 2008 16:03:59 +0200] rev 26528
Why XML notation?
wenzelm [Thu, 03 Apr 2008 16:03:57 +0200] rev 26527
Symbol.STX, Symbol.DEL;
wenzelm [Thu, 03 Apr 2008 16:03:56 +0200] rev 26526
Symbol.SOH;
wenzelm [Thu, 03 Apr 2008 16:03:55 +0200] rev 26525
added detect;
removed auxiliary buffer_of_tree;
tuned;
wenzelm [Thu, 03 Apr 2008 16:03:54 +0200] rev 26524
added some ASCII control symbols;
wenzelm [Thu, 03 Apr 2008 16:03:54 +0200] rev 26523
added Pure/General/yxml.ML;
urbanc [Thu, 03 Apr 2008 11:48:48 +0200] rev 26522
added generalised definitions for freshness of sets of atoms
and lists of atoms
haftmann [Wed, 02 Apr 2008 15:58:57 +0200] rev 26521
tuned imports
haftmann [Wed, 02 Apr 2008 15:58:43 +0200] rev 26520
tuned
haftmann [Wed, 02 Apr 2008 15:58:42 +0200] rev 26519
subst_alias
haftmann [Wed, 02 Apr 2008 15:58:41 +0200] rev 26518
improved improvements for instantiaton
haftmann [Wed, 02 Apr 2008 15:58:40 +0200] rev 26517
canonical meet_sort operation
haftmann [Wed, 02 Apr 2008 15:58:38 +0200] rev 26516
removed obscure "attach" feature
haftmann [Wed, 02 Apr 2008 15:58:37 +0200] rev 26515
extended
haftmann [Wed, 02 Apr 2008 15:58:36 +0200] rev 26514
tuned towards code generation
haftmann [Wed, 02 Apr 2008 15:58:32 +0200] rev 26513
explicit class "eq" for operational equality
haftmann [Wed, 02 Apr 2008 15:58:31 +0200] rev 26512
proofs adjusted to new situation in Int.thy/Presburger.thy
haftmann [Wed, 02 Apr 2008 15:58:30 +0200] rev 26511
explicit instantiation
haftmann [Wed, 02 Apr 2008 15:58:29 +0200] rev 26510
tuned proof
haftmann [Wed, 02 Apr 2008 15:58:28 +0200] rev 26509
dropped wrong code lemma
haftmann [Wed, 02 Apr 2008 15:58:27 +0200] rev 26508
moved some code lemmas for Numerals to other theories
haftmann [Wed, 02 Apr 2008 15:58:26 +0200] rev 26507
moved some code lemmas for Numerals here
chaieb [Wed, 02 Apr 2008 12:32:53 +0200] rev 26506
No longer imports InfiniteSet, ATP_Linkup is sufficient.
gagern [Mon, 31 Mar 2008 23:29:36 +0200] rev 26505
Catching up with smlnj.ML 1.47 (use_file), 1.52 (line numbers), 1.53
(forget_structure); doing some more advanced file name rewriting.
wenzelm [Mon, 31 Mar 2008 23:08:55 +0200] rev 26504
before close: Exn.capture/release;
wenzelm [Mon, 31 Mar 2008 23:08:54 +0200] rev 26503
discontinued unused hooks explode_platform_path_fn, platform_path_fn, shell_path_fn;
norm_absolute: non-critical (not thread-safe!);
added open_input, open_output, open_append combinators;
tuned;
wenzelm [Mon, 31 Mar 2008 23:08:53 +0200] rev 26502
added add_substring;
output: operate directly on stream;
tuned;
wenzelm [Mon, 31 Mar 2008 23:08:51 +0200] rev 26501
discontinued File.explode_platform_path -- use plain Path.explode;
nipkow [Sun, 30 Mar 2008 23:17:55 +0200] rev 26500
*** empty log message ***
wenzelm [Sat, 29 Mar 2008 22:56:01 +0100] rev 26499
functional theory setup -- requires linear access;
wenzelm [Sat, 29 Mar 2008 22:56:00 +0100] rev 26498
simplified print_simpset;
wenzelm [Sat, 29 Mar 2008 22:55:57 +0100] rev 26497
purely functional setup of claset/simpset/clasimpset;
tuned signature;
wenzelm [Sat, 29 Mar 2008 22:55:49 +0100] rev 26496
purely functional setup of claset/simpset/clasimpset;
wenzelm [Sat, 29 Mar 2008 19:24:57 +0100] rev 26495
fixed spelling;
wenzelm [Sat, 29 Mar 2008 19:14:16 +0100] rev 26494
added exec_file;
tuned;
wenzelm [Sat, 29 Mar 2008 19:14:15 +0100] rev 26493
CRITICAL: further trace levels for 1000ms and 100ms;
wenzelm [Sat, 29 Mar 2008 19:14:14 +0100] rev 26492
removed obsolete store_thm(s), cf. functional versions in pure_thy.ML;
tuned;
wenzelm [Sat, 29 Mar 2008 19:14:13 +0100] rev 26491
added generic_theory transaction;
wenzelm [Sat, 29 Mar 2008 19:14:12 +0100] rev 26490
commands 'use' and 'ML' now thy_decl;
removed obsolete 'ML_setup' -- superceded by 'ML';