Sat, 16 Feb 2008 16:43:54 +0100 System shell processes, with static input/output and propagation of interrupts.
wenzelm [Sat, 16 Feb 2008 16:43:54 +0100] rev 26078
System shell processes, with static input/output and propagation of interrupts.
Sat, 16 Feb 2008 16:43:53 +0100 added General/system_process.ML;
wenzelm [Sat, 16 Feb 2008 16:43:53 +0100] rev 26077
added General/system_process.ML;
Sat, 16 Feb 2008 02:08:07 +0100 added lemma lists {normalize,succ,pred,minus,add,mult}_bin_simps
huffman [Sat, 16 Feb 2008 02:08:07 +0100] rev 26076
added lemma lists {normalize,succ,pred,minus,add,mult}_bin_simps
Sat, 16 Feb 2008 02:01:13 +0100 added lemma lists {normalize,succ,pred,minus,add,mult}_bin_simps
huffman [Sat, 16 Feb 2008 02:01:13 +0100] rev 26075
added lemma lists {normalize,succ,pred,minus,add,mult}_bin_simps
Fri, 15 Feb 2008 23:22:02 +0100 support for managed external processes;
wenzelm [Fri, 15 Feb 2008 23:22:02 +0100] rev 26074
support for managed external processes;
Fri, 15 Feb 2008 17:36:21 +0100 more lemmas
nipkow [Fri, 15 Feb 2008 17:36:21 +0100] rev 26073
more lemmas
Fri, 15 Feb 2008 16:09:12 +0100 <= and < on nat no longer depend on wellfounded relations
haftmann [Fri, 15 Feb 2008 16:09:12 +0100] rev 26072
<= and < on nat no longer depend on wellfounded relations
Fri, 15 Feb 2008 16:09:10 +0100 moved *_reorient lemmas here
haftmann [Fri, 15 Feb 2008 16:09:10 +0100] rev 26071
moved *_reorient lemmas here
Fri, 15 Feb 2008 14:20:51 +0100 tuned names;
wenzelm [Fri, 15 Feb 2008 14:20:51 +0100] rev 26070
tuned names;
Thu, 14 Feb 2008 21:33:44 +0100 syntax error: suppress expected categories altogether;
wenzelm [Thu, 14 Feb 2008 21:33:44 +0100] rev 26069
syntax error: suppress expected categories altogether;
Thu, 14 Feb 2008 15:45:26 +0100 expected syntax categories: reduced duplication, report minimal priorities only;
wenzelm [Thu, 14 Feb 2008 15:45:26 +0100] rev 26068
expected syntax categories: reduced duplication, report minimal priorities only;
Thu, 14 Feb 2008 01:31:30 +0100 Fixed typing problem that caused instantiation of induct_aux_rec to go wrong.
berghofe [Thu, 14 Feb 2008 01:31:30 +0100] rev 26067
Fixed typing problem that caused instantiation of induct_aux_rec to go wrong.
Wed, 13 Feb 2008 15:14:17 +0100 make_meta_clause bugfix: now works for higher-order clauses like LeastI_ex
paulson [Wed, 13 Feb 2008 15:14:17 +0100] rev 26066
make_meta_clause bugfix: now works for higher-order clauses like LeastI_ex
Wed, 13 Feb 2008 10:19:30 +0100 fixed record pretty printing
kleing [Wed, 13 Feb 2008 10:19:30 +0100] rev 26065
fixed record pretty printing
Wed, 13 Feb 2008 09:35:33 +0100 using integers for pattern matching
haftmann [Wed, 13 Feb 2008 09:35:33 +0100] rev 26064
using integers for pattern matching
Wed, 13 Feb 2008 09:35:32 +0100 tuned whitespace
haftmann [Wed, 13 Feb 2008 09:35:32 +0100] rev 26063
tuned whitespace
Wed, 13 Feb 2008 09:35:31 +0100 more abstract lemmas
haftmann [Wed, 13 Feb 2008 09:35:31 +0100] rev 26062
more abstract lemmas
Mon, 11 Feb 2008 22:12:19 +0100 fix spelling
huffman [Mon, 11 Feb 2008 22:12:19 +0100] rev 26061
fix spelling
Mon, 11 Feb 2008 21:32:13 +0100 imports Main;
wenzelm [Mon, 11 Feb 2008 21:32:13 +0100] rev 26060
imports Main;
Mon, 11 Feb 2008 21:32:12 +0100 removed unnecessary theory qualifiers;
wenzelm [Mon, 11 Feb 2008 21:32:12 +0100] rev 26059
removed unnecessary theory qualifiers;
Mon, 11 Feb 2008 21:32:11 +0100 simultaneous use_thys;
wenzelm [Mon, 11 Feb 2008 21:32:11 +0100] rev 26058
simultaneous use_thys;
Mon, 11 Feb 2008 21:32:10 +0100 added Id;
wenzelm [Mon, 11 Feb 2008 21:32:10 +0100] rev 26057
added Id;
Mon, 11 Feb 2008 15:40:21 +0100 Made theory names in ZF disjoint from HOL theory names to allow loading both developments
krauss [Mon, 11 Feb 2008 15:40:21 +0100] rev 26056
Made theory names in ZF disjoint from HOL theory names to allow loading both developments in a single session (but not merge them).
Mon, 11 Feb 2008 15:19:17 +0100 tuned proofs and comments
urbanc [Mon, 11 Feb 2008 15:19:17 +0100] rev 26055
tuned proofs and comments
Sun, 10 Feb 2008 20:49:48 +0100 tuned spaces;
wenzelm [Sun, 10 Feb 2008 20:49:48 +0100] rev 26054
tuned spaces;
Sun, 10 Feb 2008 20:49:47 +0100 tuned default position;
wenzelm [Sun, 10 Feb 2008 20:49:47 +0100] rev 26053
tuned default position;
Sun, 10 Feb 2008 20:49:46 +0100 added default_properties;
wenzelm [Sun, 10 Feb 2008 20:49:46 +0100] rev 26052
added default_properties;
Sun, 10 Feb 2008 20:49:45 +0100 added position_properties;
wenzelm [Sun, 10 Feb 2008 20:49:45 +0100] rev 26051
added position_properties;
Sun, 10 Feb 2008 20:49:42 +0100 maintain default position;
wenzelm [Sun, 10 Feb 2008 20:49:42 +0100] rev 26050
maintain default position;
Sat, 09 Feb 2008 12:56:12 +0100 overloading: reduced code redundancy, no xstrings here;
wenzelm [Sat, 09 Feb 2008 12:56:12 +0100] rev 26049
overloading: reduced code redundancy, no xstrings here;
(0) -10000 -3000 -1000 -300 -100 -50 -30 +30 +50 +100 +300 +1000 +3000 +10000 +30000 tip