Fri, 30 Mar 2012 14:25:32 +0200 rephrase lemmas about arithmetic series using numeral '2'
huffman [Fri, 30 Mar 2012 14:25:32 +0200] rev 47222
rephrase lemmas about arithmetic series using numeral '2'
Fri, 30 Mar 2012 14:00:18 +0200 rephrase lemma card_Pow using '2' instead of 'Suc (Suc 0)'
huffman [Fri, 30 Mar 2012 14:00:18 +0200] rev 47221
rephrase lemma card_Pow using '2' instead of 'Suc (Suc 0)'
Fri, 30 Mar 2012 12:32:35 +0200 replace lemmas eval_nat_numeral with a simpler reformulation
huffman [Fri, 30 Mar 2012 12:32:35 +0200] rev 47220
replace lemmas eval_nat_numeral with a simpler reformulation
Fri, 30 Mar 2012 12:02:23 +0200 restate various simp rules for word operations using pred_numeral
huffman [Fri, 30 Mar 2012 12:02:23 +0200] rev 47219
restate various simp rules for word operations using pred_numeral
Fri, 30 Mar 2012 11:52:26 +0200 new lemmas for simplifying subtraction on nat numerals
huffman [Fri, 30 Mar 2012 11:52:26 +0200] rev 47218
new lemmas for simplifying subtraction on nat numerals
Fri, 30 Mar 2012 11:16:35 +0200 removed redundant nat-specific copies of theorems
huffman [Fri, 30 Mar 2012 11:16:35 +0200] rev 47217
removed redundant nat-specific copies of theorems
Fri, 30 Mar 2012 10:41:27 +0200 move more theorems from Nat_Numeral.thy to Num.thy
huffman [Fri, 30 Mar 2012 10:41:27 +0200] rev 47216
move more theorems from Nat_Numeral.thy to Num.thy
Fri, 30 Mar 2012 15:25:47 +0200 "invariant" is free in main HOL (cf. 56adbf5bcc82, e64ffc96a49f);
wenzelm [Fri, 30 Mar 2012 15:25:47 +0200] rev 47215
"invariant" is free in main HOL (cf. 56adbf5bcc82, e64ffc96a49f);
Fri, 30 Mar 2012 13:12:02 +0200 more robust ISABELLE_JDK_HOME settings, based on exisiting JAVA_HOME provided by isatest shell environment (which depends a lot on the host);
wenzelm [Fri, 30 Mar 2012 13:12:02 +0200] rev 47214
more robust ISABELLE_JDK_HOME settings, based on exisiting JAVA_HOME provided by isatest shell environment (which depends a lot on the host);
Fri, 30 Mar 2012 11:48:24 +0200 more explicit isatest environment settings (from private .bashrc);
wenzelm [Fri, 30 Mar 2012 11:48:24 +0200] rev 47213
more explicit isatest environment settings (from private .bashrc);
Fri, 30 Mar 2012 09:55:03 +0200 merged
huffman [Fri, 30 Mar 2012 09:55:03 +0200] rev 47212
merged
Fri, 30 Mar 2012 08:15:29 +0200 fix search-and-replace errors
huffman [Fri, 30 Mar 2012 08:15:29 +0200] rev 47211
fix search-and-replace errors
Fri, 30 Mar 2012 08:04:28 +0200 move lemma card_UNIV_bool from Nat_Numeral.thy to Finite_Set.thy
huffman [Fri, 30 Mar 2012 08:04:28 +0200] rev 47210
move lemma card_UNIV_bool from Nat_Numeral.thy to Finite_Set.thy
Fri, 30 Mar 2012 09:08:29 +0200 add constant pred_numeral k = numeral k - (1::nat);
huffman [Fri, 30 Mar 2012 09:08:29 +0200] rev 47209
add constant pred_numeral k = numeral k - (1::nat); replace several simp rules from Nat_Numeral.thy with new ones that use pred_numeral
Fri, 30 Mar 2012 08:11:52 +0200 move lemmas from Nat_Numeral.thy to Nat.thy
huffman [Fri, 30 Mar 2012 08:11:52 +0200] rev 47208
move lemmas from Nat_Numeral.thy to Nat.thy
Fri, 30 Mar 2012 08:10:28 +0200 move lemmas from Nat_Numeral to Int.thy and Num.thy
huffman [Fri, 30 Mar 2012 08:10:28 +0200] rev 47207
move lemmas from Nat_Numeral to Int.thy and Num.thy
Fri, 30 Mar 2012 09:32:18 +0200 merged
bulwahn [Fri, 30 Mar 2012 09:32:18 +0200] rev 47206
merged
Fri, 30 Mar 2012 08:44:01 +0200 adding theory to prove completeness of the exhaustive generators
bulwahn [Fri, 30 Mar 2012 08:44:01 +0200] rev 47205
adding theory to prove completeness of the exhaustive generators
Fri, 30 Mar 2012 08:19:31 +0200 refine bindings in quickcheck_common: do not conceal and do not declare as simps
bulwahn [Fri, 30 Mar 2012 08:19:31 +0200] rev 47204
refine bindings in quickcheck_common: do not conceal and do not declare as simps
Fri, 30 Mar 2012 08:19:29 +0200 hiding fact not so aggressively
bulwahn [Fri, 30 Mar 2012 08:19:29 +0200] rev 47203
hiding fact not so aggressively
Fri, 30 Mar 2012 09:04:29 +0200 power on predicate relations
haftmann [Fri, 30 Mar 2012 09:04:29 +0200] rev 47202
power on predicate relations
Fri, 30 Mar 2012 00:01:30 +0100 made Mirabelle-SH's 'trivial' check optional;
sultana [Fri, 30 Mar 2012 00:01:30 +0100] rev 47201
made Mirabelle-SH's 'trivial' check optional;
Thu, 29 Mar 2012 22:52:24 +0200 merged
wenzelm [Thu, 29 Mar 2012 22:52:24 +0200] rev 47200
merged
Thu, 29 Mar 2012 22:43:50 +0200 more specific notion of partiality (cf. Scala version);
wenzelm [Thu, 29 Mar 2012 22:43:50 +0200] rev 47199
more specific notion of partiality (cf. Scala version);
Thu, 29 Mar 2012 21:13:48 +0200 use qualified names for rsp and rep_eq theorems in quotient_def
kuncar [Thu, 29 Mar 2012 21:13:48 +0200] rev 47198
use qualified names for rsp and rep_eq theorems in quotient_def
Thu, 29 Mar 2012 17:40:44 +0200 announcing NEWS (cf. 446cfc760ccf)
bulwahn [Thu, 29 Mar 2012 17:40:44 +0200] rev 47197
announcing NEWS (cf. 446cfc760ccf)
Thu, 29 Mar 2012 14:47:31 +0200 remove obsolete simp rule for powers
huffman [Thu, 29 Mar 2012 14:47:31 +0200] rev 47196
remove obsolete simp rule for powers
Thu, 29 Mar 2012 14:42:55 +0200 remove duplicate lemmas power_m1_{even,odd} in favor of power_minus1_{even,odd}
huffman [Thu, 29 Mar 2012 14:42:55 +0200] rev 47195
remove duplicate lemmas power_m1_{even,odd} in favor of power_minus1_{even,odd}
Thu, 29 Mar 2012 14:39:05 +0200 remove unneeded rewrite rules for powers of numerals
huffman [Thu, 29 Mar 2012 14:39:05 +0200] rev 47194
remove unneeded rewrite rules for powers of numerals
Thu, 29 Mar 2012 14:29:36 +0200 remove duplicate lemma Suc_numeral
huffman [Thu, 29 Mar 2012 14:29:36 +0200] rev 47193
remove duplicate lemma Suc_numeral
Thu, 29 Mar 2012 14:09:10 +0200 move many lemmas from Nat_Numeral.thy to Power.thy or Num.thy
huffman [Thu, 29 Mar 2012 14:09:10 +0200] rev 47192
move many lemmas from Nat_Numeral.thy to Power.thy or Num.thy
Thu, 29 Mar 2012 11:47:30 +0200 bootstrap Num.thy before Power.thy;
huffman [Thu, 29 Mar 2012 11:47:30 +0200] rev 47191
bootstrap Num.thy before Power.thy; move lemmas about powers into Power.thy
Thu, 29 Mar 2012 08:59:56 +0200 educated guess to include jdk
haftmann [Thu, 29 Mar 2012 08:59:56 +0200] rev 47190
educated guess to include jdk
Wed, 28 Mar 2012 17:57:23 +0200 improved robustness with new antiquoation by Makarius
nipkow [Wed, 28 Mar 2012 17:57:23 +0200] rev 47189
improved robustness with new antiquoation by Makarius
Wed, 28 Mar 2012 16:12:17 +0200 merged
nipkow [Wed, 28 Mar 2012 16:12:17 +0200] rev 47188
merged
Wed, 28 Mar 2012 16:12:10 +0200 updates
nipkow [Wed, 28 Mar 2012 16:12:10 +0200] rev 47187
updates
Wed, 28 Mar 2012 14:54:33 +0200 updated documentation files (cf. c14fda8fee38)
bulwahn [Wed, 28 Mar 2012 14:54:33 +0200] rev 47186
updated documentation files (cf. c14fda8fee38)
Wed, 28 Mar 2012 13:53:30 +0200 clarified ISABELLE_JDK_HOME: derive from running JVM, but ignore accidental JAVA_HOME;
wenzelm [Wed, 28 Mar 2012 13:53:30 +0200] rev 47185
clarified ISABELLE_JDK_HOME: derive from running JVM, but ignore accidental JAVA_HOME; clarified jEdit/README_BUILD;
Wed, 28 Mar 2012 13:38:56 +0200 merged
wenzelm [Wed, 28 Mar 2012 13:38:56 +0200] rev 47184
merged
Wed, 28 Mar 2012 12:28:24 +0200 removed references to obsolete theorems
huffman [Wed, 28 Mar 2012 12:28:24 +0200] rev 47183
removed references to obsolete theorems
Wed, 28 Mar 2012 11:40:12 +0200 merged
bulwahn [Wed, 28 Mar 2012 11:40:12 +0200] rev 47182
merged
Wed, 28 Mar 2012 10:44:04 +0200 some tuning while reviewing the current state of the quotient_def package
bulwahn [Wed, 28 Mar 2012 10:44:04 +0200] rev 47181
some tuning while reviewing the current state of the quotient_def package
Wed, 28 Mar 2012 10:37:30 +0200 improving spelling
bulwahn [Wed, 28 Mar 2012 10:37:30 +0200] rev 47180
improving spelling
Wed, 28 Mar 2012 10:16:02 +0200 changing more definitions to quotient_definition
bulwahn [Wed, 28 Mar 2012 10:16:02 +0200] rev 47179
changing more definitions to quotient_definition
Wed, 28 Mar 2012 10:02:22 +0200 removing now redundant impl_of theorems in DAList
bulwahn [Wed, 28 Mar 2012 10:02:22 +0200] rev 47178
removing now redundant impl_of theorems in DAList
Wed, 28 Mar 2012 10:00:52 +0200 using abstract code equations for proofs of code equations in Multiset
bulwahn [Wed, 28 Mar 2012 10:00:52 +0200] rev 47177
using abstract code equations for proofs of code equations in Multiset
Wed, 28 Mar 2012 12:08:08 +0200 simplified statements and proofs;
wenzelm [Wed, 28 Mar 2012 12:08:08 +0200] rev 47176
simplified statements and proofs;
Wed, 28 Mar 2012 11:46:14 +0200 tuned whitespace;
wenzelm [Wed, 28 Mar 2012 11:46:14 +0200] rev 47175
tuned whitespace;
Wed, 28 Mar 2012 11:17:32 +0200 updated Sign.add_type, Name_Space.declare;
wenzelm [Wed, 28 Mar 2012 11:17:32 +0200] rev 47174
updated Sign.add_type, Name_Space.declare;
Wed, 28 Mar 2012 11:04:39 +0200 updated comments;
wenzelm [Wed, 28 Mar 2012 11:04:39 +0200] rev 47173
updated comments;
Wed, 28 Mar 2012 08:25:51 +0200 merged
huffman [Wed, 28 Mar 2012 08:25:51 +0200] rev 47172
merged
Tue, 27 Mar 2012 22:10:26 +0200 remove unnecessary rules from the simpset
huffman [Tue, 27 Mar 2012 22:10:26 +0200] rev 47171
remove unnecessary rules from the simpset
Tue, 27 Mar 2012 21:58:41 +0200 remove unused premises
huffman [Tue, 27 Mar 2012 21:58:41 +0200] rev 47170
remove unused premises
Tue, 27 Mar 2012 21:48:55 +0200 remove duplicate lemmas
huffman [Tue, 27 Mar 2012 21:48:55 +0200] rev 47169
remove duplicate lemmas
Tue, 27 Mar 2012 21:48:26 +0200 mark some duplicate lemmas for deletion
huffman [Tue, 27 Mar 2012 21:48:26 +0200] rev 47168
mark some duplicate lemmas for deletion
Tue, 27 Mar 2012 20:19:23 +0200 remove more redundant lemmas
huffman [Tue, 27 Mar 2012 20:19:23 +0200] rev 47167
remove more redundant lemmas
Tue, 27 Mar 2012 16:49:23 +0200 tuned proofs
huffman [Tue, 27 Mar 2012 16:49:23 +0200] rev 47166
tuned proofs
Tue, 27 Mar 2012 19:21:05 +0200 remove redundant lemmas
huffman [Tue, 27 Mar 2012 19:21:05 +0200] rev 47165
remove redundant lemmas
Tue, 27 Mar 2012 16:04:51 +0200 generalized lemma zpower_zmod
huffman [Tue, 27 Mar 2012 16:04:51 +0200] rev 47164
generalized lemma zpower_zmod
Tue, 27 Mar 2012 15:53:48 +0200 remove redundant lemma
huffman [Tue, 27 Mar 2012 15:53:48 +0200] rev 47163
remove redundant lemma
Tue, 27 Mar 2012 15:40:11 +0200 remove redundant lemma
huffman [Tue, 27 Mar 2012 15:40:11 +0200] rev 47162
remove redundant lemma
Tue, 27 Mar 2012 15:34:36 +0200 remove duplicate [algebra] declarations
huffman [Tue, 27 Mar 2012 15:34:36 +0200] rev 47161
remove duplicate [algebra] declarations
Tue, 27 Mar 2012 15:34:04 +0200 generalize more div/mod lemmas
huffman [Tue, 27 Mar 2012 15:34:04 +0200] rev 47160
generalize more div/mod lemmas
Tue, 27 Mar 2012 15:27:49 +0200 generalize some theorems about div/mod
huffman [Tue, 27 Mar 2012 15:27:49 +0200] rev 47159
generalize some theorems about div/mod
Wed, 28 Mar 2012 00:18:11 +0200 updated to jedit-4.5.1;
wenzelm [Wed, 28 Mar 2012 00:18:11 +0200] rev 47158
updated to jedit-4.5.1;
Tue, 27 Mar 2012 17:58:53 +0200 merged
kuncar [Tue, 27 Mar 2012 17:58:53 +0200] rev 47157
merged
Tue, 27 Mar 2012 14:46:34 +0200 note a code eqn in quotient_def
kuncar [Tue, 27 Mar 2012 14:46:34 +0200] rev 47156
note a code eqn in quotient_def
Tue, 27 Mar 2012 17:11:02 +0200 dropped support for List.distinct in binding to SMT solvers: only few applications benefited from this support, and in some cases the smt method fails due to its support for List.distinct
boehmes [Tue, 27 Mar 2012 17:11:02 +0200] rev 47155
dropped support for List.distinct in binding to SMT solvers: only few applications benefited from this support, and in some cases the smt method fails due to its support for List.distinct
Tue, 27 Mar 2012 16:59:13 +0300 more robustness in case a theorem cannot be retrieved (which typically happens with backtick facts)
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47154
more robustness in case a theorem cannot be retrieved (which typically happens with backtick facts)
Tue, 27 Mar 2012 16:59:13 +0300 fixed eta-extension of higher-order quantifiers in THF output
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47153
fixed eta-extension of higher-order quantifiers in THF output
Tue, 27 Mar 2012 16:59:13 +0300 renamed "smt_fixed" to "smt_read_only_certificates"
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47152
renamed "smt_fixed" to "smt_read_only_certificates"
Tue, 27 Mar 2012 16:59:13 +0300 tuning
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47151
tuning
Tue, 27 Mar 2012 16:59:13 +0300 tuning (in particular, Symtab instead of AList)
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47150
tuning (in particular, Symtab instead of AList)
Tue, 27 Mar 2012 16:59:13 +0300 tweak slices, based on eval by Daniel Wand
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47149
tweak slices, based on eval by Daniel Wand
Tue, 27 Mar 2012 16:59:13 +0300 be less forceful about ":lt" to make infinite loops less likely (could still fail with mutually recursive tail rec functions)
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47148
be less forceful about ":lt" to make infinite loops less likely (could still fail with mutually recursive tail rec functions)
Tue, 27 Mar 2012 16:59:13 +0300 print a hint
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47147
print a hint
Tue, 27 Mar 2012 16:59:13 +0300 avoid DL
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47146
avoid DL
Tue, 27 Mar 2012 16:59:13 +0300 TFF: declare free types as types
blanchet [Tue, 27 Mar 2012 16:59:13 +0300] rev 47145
TFF: declare free types as types
Tue, 27 Mar 2012 15:34:04 +0200 merged
bulwahn [Tue, 27 Mar 2012 15:34:04 +0200] rev 47144
merged
Tue, 27 Mar 2012 14:14:46 +0200 association lists with distinct keys uses the quotient infrastructure to obtain code certificates;
bulwahn [Tue, 27 Mar 2012 14:14:46 +0200] rev 47143
association lists with distinct keys uses the quotient infrastructure to obtain code certificates; added remarks about further improvements
Tue, 27 Mar 2012 14:49:56 +0200 remove redundant lemmas
huffman [Tue, 27 Mar 2012 14:49:56 +0200] rev 47142
remove redundant lemmas
Tue, 27 Mar 2012 12:42:54 +0200 move int::ring_div instance upward, simplify several proofs
huffman [Tue, 27 Mar 2012 12:42:54 +0200] rev 47141
move int::ring_div instance upward, simplify several proofs
Tue, 27 Mar 2012 11:45:02 +0200 rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
huffman [Tue, 27 Mar 2012 11:45:02 +0200] rev 47140
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
Tue, 27 Mar 2012 11:41:16 +0200 extend definition of divmod_int_rel to handle denominator=0 case
huffman [Tue, 27 Mar 2012 11:41:16 +0200] rev 47139
extend definition of divmod_int_rel to handle denominator=0 case
Tue, 27 Mar 2012 11:02:18 +0200 tuned proofs
huffman [Tue, 27 Mar 2012 11:02:18 +0200] rev 47138
tuned proofs
Tue, 27 Mar 2012 10:34:12 +0200 shorten a proof
huffman [Tue, 27 Mar 2012 10:34:12 +0200] rev 47137
shorten a proof
Tue, 27 Mar 2012 10:20:31 +0200 simplify some proofs
huffman [Tue, 27 Mar 2012 10:20:31 +0200] rev 47136
simplify some proofs
Tue, 27 Mar 2012 09:54:39 +0200 rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
huffman [Tue, 27 Mar 2012 09:54:39 +0200] rev 47135
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
Tue, 27 Mar 2012 09:44:56 +0200 simplify some proofs
huffman [Tue, 27 Mar 2012 09:44:56 +0200] rev 47134
simplify some proofs
Mon, 26 Mar 2012 21:03:30 +0200 merged
wenzelm [Mon, 26 Mar 2012 21:03:30 +0200] rev 47133
merged
Mon, 26 Mar 2012 21:00:39 +0200 merged
nipkow [Mon, 26 Mar 2012 21:00:39 +0200] rev 47132
merged
Mon, 26 Mar 2012 21:00:23 +0200 reverted to canonical name
nipkow [Mon, 26 Mar 2012 21:00:23 +0200] rev 47131
reverted to canonical name
Mon, 26 Mar 2012 20:45:59 +0200 merged
wenzelm [Mon, 26 Mar 2012 20:45:59 +0200] rev 47130
merged
Mon, 26 Mar 2012 20:11:27 +0200 merged
huffman [Mon, 26 Mar 2012 20:11:27 +0200] rev 47129
merged
Mon, 26 Mar 2012 20:09:18 +0200 revert changeset 500a5d97511a, re-enabling HOL-Proofs-Lambda
huffman [Mon, 26 Mar 2012 20:09:18 +0200] rev 47128
revert changeset 500a5d97511a, re-enabling HOL-Proofs-Lambda
Mon, 26 Mar 2012 20:07:41 +0200 merged
huffman [Mon, 26 Mar 2012 20:07:41 +0200] rev 47127
merged
Mon, 26 Mar 2012 20:07:29 +0200 fix incorrect code_modulename declarations
huffman [Mon, 26 Mar 2012 20:07:29 +0200] rev 47126
fix incorrect code_modulename declarations
Mon, 26 Mar 2012 19:04:17 +0200 code lemma for function 'nat' that doesn't go into an infinite loop (fixes problem with non-terminating HOL-Proofs-Lambda)
huffman [Mon, 26 Mar 2012 19:04:17 +0200] rev 47125
code lemma for function 'nat' that doesn't go into an infinite loop (fixes problem with non-terminating HOL-Proofs-Lambda)
Mon, 26 Mar 2012 19:03:27 +0200 remove old-style semicolon
huffman [Mon, 26 Mar 2012 19:03:27 +0200] rev 47124
remove old-style semicolon
Mon, 26 Mar 2012 20:09:52 +0200 merged
nipkow [Mon, 26 Mar 2012 20:09:52 +0200] rev 47123
merged
Mon, 26 Mar 2012 18:54:41 +0200 Functions and lemmas by Christian Sternagel
nipkow [Mon, 26 Mar 2012 18:54:41 +0200] rev 47122
Functions and lemmas by Christian Sternagel
Mon, 26 Mar 2012 20:42:00 +0200 more precise treatment of \r\n as blank symbol (cf. 2bf29095d26f), e.g. relevant for loading theory headers in Isabelle/jEdit -- NB: jEdit and Isabelle/ML normalize newline variants to \n, but Isabelle/Scala retains them literally;
wenzelm [Mon, 26 Mar 2012 20:42:00 +0200] rev 47121
more precise treatment of \r\n as blank symbol (cf. 2bf29095d26f), e.g. relevant for loading theory headers in Isabelle/jEdit -- NB: jEdit and Isabelle/ML normalize newline variants to \n, but Isabelle/Scala retains them literally;
Mon, 26 Mar 2012 19:18:03 +0200 disabled HOL-Proofs-Lambda temporarily, which causes problems with 2a1953f0d20d;
wenzelm [Mon, 26 Mar 2012 19:18:03 +0200] rev 47120
disabled HOL-Proofs-Lambda temporarily, which causes problems with 2a1953f0d20d;
Mon, 26 Mar 2012 18:32:22 +0200 tuned comment
kuncar [Mon, 26 Mar 2012 18:32:22 +0200] rev 47119
tuned comment
Mon, 26 Mar 2012 17:58:47 +0200 merged
kuncar [Mon, 26 Mar 2012 17:58:47 +0200] rev 47118
merged
Mon, 26 Mar 2012 15:33:28 +0200 merged
kuncar [Mon, 26 Mar 2012 15:33:28 +0200] rev 47117
merged
Mon, 26 Mar 2012 15:32:54 +0200 tuned proof - no smt call
kuncar [Mon, 26 Mar 2012 15:32:54 +0200] rev 47116
tuned proof - no smt call
Mon, 26 Mar 2012 16:25:08 +0200 more robust command invocation via ISABELLE_JDK_HOME or SCALA_HOME (NB: bash exec requires genuine executable, not function);
wenzelm [Mon, 26 Mar 2012 16:25:08 +0200] rev 47115
more robust command invocation via ISABELLE_JDK_HOME or SCALA_HOME (NB: bash exec requires genuine executable, not function);
Mon, 26 Mar 2012 15:38:09 +0200 updated theory header syntax and related details;
wenzelm [Mon, 26 Mar 2012 15:38:09 +0200] rev 47114
updated theory header syntax and related details;
Sat, 24 Mar 2012 20:24:16 +0100 ISABELLE_JDK_HOME settings variable points to JDK with javac and jar (not just JRE);
wenzelm [Sat, 24 Mar 2012 20:24:16 +0100] rev 47113
ISABELLE_JDK_HOME settings variable points to JDK with javac and jar (not just JRE); update for prospective jdk1.7.x component;
Mon, 26 Mar 2012 11:15:41 +0200 merged
wenzelm [Mon, 26 Mar 2012 11:15:41 +0200] rev 47112
merged
Mon, 26 Mar 2012 11:01:04 +0200 reintroduced broken proofs and regenerated certificates
blanchet [Mon, 26 Mar 2012 11:01:04 +0200] rev 47111
reintroduced broken proofs and regenerated certificates
Mon, 26 Mar 2012 10:56:56 +0200 merged, resolving trivial conflict;
wenzelm [Mon, 26 Mar 2012 10:56:56 +0200] rev 47110
merged, resolving trivial conflict;
Mon, 26 Mar 2012 10:42:06 +0200 fixed Nitpick after numeral representation change (2a1953f0d20d)
blanchet [Mon, 26 Mar 2012 10:42:06 +0200] rev 47109
fixed Nitpick after numeral representation change (2a1953f0d20d)
Sun, 25 Mar 2012 20:15:39 +0200 merged fork with new numeral representation (see NEWS)
huffman [Sun, 25 Mar 2012 20:15:39 +0200] rev 47108
merged fork with new numeral representation (see NEWS)
Sat, 24 Mar 2012 16:27:04 +0100 merged
kuncar [Sat, 24 Mar 2012 16:27:04 +0100] rev 47107
merged
Fri, 23 Mar 2012 22:00:17 +0100 use Thm.transfer for thms stored in generic context data storage
kuncar [Fri, 23 Mar 2012 22:00:17 +0100] rev 47106
use Thm.transfer for thms stored in generic context data storage
Fri, 23 Mar 2012 18:23:47 +0100 hide invariant constant
kuncar [Fri, 23 Mar 2012 18:23:47 +0100] rev 47105
hide invariant constant
Sat, 24 Mar 2012 12:28:45 +0100 explicit SMTP server (appears to be required after recent change of system configuration);
wenzelm [Sat, 24 Mar 2012 12:28:45 +0100] rev 47104
explicit SMTP server (appears to be required after recent change of system configuration);
Sat, 24 Mar 2012 12:22:29 +0100 more isatest subscribers;
wenzelm [Sat, 24 Mar 2012 12:22:29 +0100] rev 47103
more isatest subscribers;
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip