haftmann [Fri, 23 Feb 2007 08:39:21 +0100] rev 22348
adjusted code lemmas
haftmann [Fri, 23 Feb 2007 08:39:20 +0100] rev 22347
continued
haftmann [Fri, 23 Feb 2007 08:39:19 +0100] rev 22346
dropped diagnostic switch
paulson [Thu, 22 Feb 2007 10:25:14 +0100] rev 22345
Improved handling of situation when theorem in cache disagrees with theorem supplied: new clauses
are now returned, fixing a bug in the metis method.
krauss [Wed, 21 Feb 2007 13:51:12 +0100] rev 22344
Fixed print translations for quantifiers a la "ALL x>=t. P x". These used
to fail when the other term in the comparison was itself a bound variable,
as in "EX y. ALL x>=y. P x".
kleing [Wed, 21 Feb 2007 02:30:06 +0100] rev 22343
prevent quadratic time removal of duplicates if filter list is empty (likely to have too many results)
kleing [Tue, 20 Feb 2007 00:53:18 +0100] rev 22342
added missing \
kleing [Tue, 20 Feb 2007 00:23:58 +0100] rev 22341
updated docs with new with_dups syntax for find_theorems
kleing [Tue, 20 Feb 2007 00:14:33 +0100] rev 22340
Remove duplicates from printed theorems in find_theorems
(still pretty slow, needs optimising).
Added syntax "find_theorems (..) with_dups .." to switch off removal.
schirmer [Mon, 19 Feb 2007 16:44:08 +0100] rev 22339
more precise error message in parameter unification
aspinall [Sat, 17 Feb 2007 18:01:22 +0100] rev 22338
Updated
aspinall [Sat, 17 Feb 2007 18:00:59 +0100] rev 22337
Fix <pgipquit>. Remove unused pgmlatomsN. Make showid match askids. Use string functions for showid, avoiding printwrap kludge.
aspinall [Sat, 17 Feb 2007 17:22:53 +0100] rev 22336
<idvalue>: add name attribute to allow unsolicited updates.
aspinall [Sat, 17 Feb 2007 17:19:59 +0100] rev 22335
pretty_full_theory: expose in signature.
aspinall [Sat, 17 Feb 2007 17:18:47 +0100] rev 22334
Clarify comment
wenzelm [Fri, 16 Feb 2007 22:46:03 +0100] rev 22333
unified arity parser/arguments;
wenzelm [Fri, 16 Feb 2007 22:13:16 +0100] rev 22332
ML text: informative Output.debug only;
wenzelm [Fri, 16 Feb 2007 22:13:15 +0100] rev 22331
unified arity parser/arguments;
berghofe [Fri, 16 Feb 2007 19:19:19 +0100] rev 22330
Replaced "raise RecError" by "primrec_err" in function
gen_primrec_i to prevent error message from being suppressed.
schirmer [Fri, 16 Feb 2007 11:01:16 +0100] rev 22329
added example for print-mode Axiom
schirmer [Fri, 16 Feb 2007 11:00:47 +0100] rev 22328
added print-mode Axiom to print theorems without premises with a rule on top.
krauss [Fri, 16 Feb 2007 09:04:23 +0100] rev 22327
updated Makefile
narboux [Thu, 15 Feb 2007 18:18:21 +0100] rev 22326
start adding the attribute eqvt to some lemmas of the nominal library
krauss [Thu, 15 Feb 2007 17:35:19 +0100] rev 22325
changed termination goal to use object quantifier
krauss [Thu, 15 Feb 2007 12:14:34 +0100] rev 22324
added congruence rule for function composition
krauss [Thu, 15 Feb 2007 12:02:11 +0100] rev 22323
beta_eta_contract specification befor processing. These normal forms avoid unpleasant surprises later on.
haftmann [Wed, 14 Feb 2007 10:07:17 +0100] rev 22322
continued
haftmann [Wed, 14 Feb 2007 10:06:17 +0100] rev 22321
class package now using Locale.interpretation_i
haftmann [Wed, 14 Feb 2007 10:06:16 +0100] rev 22320
clarified explanation
haftmann [Wed, 14 Feb 2007 10:06:15 +0100] rev 22319
cleanup
haftmann [Wed, 14 Feb 2007 10:06:14 +0100] rev 22318
simpliefied instance statement
haftmann [Wed, 14 Feb 2007 10:06:13 +0100] rev 22317
continued class tutorial
haftmann [Wed, 14 Feb 2007 10:06:12 +0100] rev 22316
added class "preorder"
berghofe [Tue, 13 Feb 2007 18:26:48 +0100] rev 22315
Added nominal_inductive keyword.
berghofe [Tue, 13 Feb 2007 18:19:25 +0100] rev 22314
Added new file Nominal/nominal_inductive.ML
berghofe [Tue, 13 Feb 2007 18:18:45 +0100] rev 22313
First steps towards strengthening of induction rules for
inductively defined predicates involving nominal datatypes.
berghofe [Tue, 13 Feb 2007 18:17:28 +0100] rev 22312
Added new file nominal_inductive.ML
berghofe [Tue, 13 Feb 2007 18:16:50 +0100] rev 22311
Curried and exported mk_perm.
paulson [Tue, 13 Feb 2007 16:37:14 +0100] rev 22310
COMP now performs a distinctness check on the multiple results before failing
bulwahn [Tue, 13 Feb 2007 10:09:21 +0100] rev 22309
improved lexicographic order termination tactic
haftmann [Sat, 10 Feb 2007 17:06:40 +0100] rev 22308
added OCaml example
paulson [Sat, 10 Feb 2007 16:43:23 +0100] rev 22307
Completing the bug fix from the previous update: the result of unifying type
variables must be normalized WRT itself; otherwise instantiation is wrong
haftmann [Sat, 10 Feb 2007 09:26:26 +0100] rev 22306
changed representation of constants; consistent name handling
haftmann [Sat, 10 Feb 2007 09:26:25 +0100] rev 22305
changed representation of constants
haftmann [Sat, 10 Feb 2007 09:26:24 +0100] rev 22304
tuned
haftmann [Sat, 10 Feb 2007 09:26:23 +0100] rev 22303
new Isar command print_codesetup
haftmann [Sat, 10 Feb 2007 09:26:22 +0100] rev 22302
added experimental class target
haftmann [Sat, 10 Feb 2007 09:26:20 +0100] rev 22301
added class target stub
haftmann [Sat, 10 Feb 2007 09:26:19 +0100] rev 22300
internal interfaces for interpretation and interpret
haftmann [Sat, 10 Feb 2007 09:26:18 +0100] rev 22299
moved commands of class package here
haftmann [Sat, 10 Feb 2007 09:26:17 +0100] rev 22298
added class package to Isar bootstrap
haftmann [Sat, 10 Feb 2007 09:26:16 +0100] rev 22297
splut up code generation in two parts
haftmann [Sat, 10 Feb 2007 09:26:15 +0100] rev 22296
canonical interface for attributes
haftmann [Sat, 10 Feb 2007 09:26:14 +0100] rev 22295
changed name of interpretation linorder to order
haftmann [Sat, 10 Feb 2007 09:26:12 +0100] rev 22294
adjusted to changes in class package
haftmann [Sat, 10 Feb 2007 09:26:11 +0100] rev 22293
added outline for Isabelle library description
haftmann [Sat, 10 Feb 2007 09:26:10 +0100] rev 22292
adjusted to new code generator Isar commands and changes in implementation
haftmann [Sat, 10 Feb 2007 09:26:09 +0100] rev 22291
adjusted to new code generator Isar commands
haftmann [Sat, 10 Feb 2007 09:26:08 +0100] rev 22290
added references for code generator tutorial
haftmann [Sat, 10 Feb 2007 09:26:07 +0100] rev 22289
added antiquotation for exceptions
haftmann [Sat, 10 Feb 2007 09:26:06 +0100] rev 22288
updated keywords
paulson [Thu, 08 Feb 2007 18:14:13 +0100] rev 22287
cterm_instantiate was calling a type instantiation function that works only for matching,
not unification as here.
urbanc [Thu, 08 Feb 2007 17:22:22 +0100] rev 22286
added get-functions
berghofe [Wed, 07 Feb 2007 18:12:58 +0100] rev 22285
Renamed member to memb to avoid confusion with member function
defined in Predicate theory.
berghofe [Wed, 07 Feb 2007 18:12:02 +0100] rev 22284
Adapted to changes in Finite_Set theory.
berghofe [Wed, 07 Feb 2007 18:11:27 +0100] rev 22283
Adapted to new inductive definition package.
berghofe [Wed, 07 Feb 2007 18:10:21 +0100] rev 22282
- Adapted to new inductive definition package
- Adapted to changes in Multiset theory
berghofe [Wed, 07 Feb 2007 18:07:10 +0100] rev 22281
Added meta_spec to extraction_expand.
berghofe [Wed, 07 Feb 2007 18:04:44 +0100] rev 22280
Added functions hhf_proof and un_hhf_proof.
berghofe [Wed, 07 Feb 2007 18:03:18 +0100] rev 22279
Adapted to changes in Accessible_Part and Wellfounded_Recursion theories.
berghofe [Wed, 07 Feb 2007 18:01:40 +0100] rev 22278
Added split_rule attribute.
berghofe [Wed, 07 Feb 2007 18:00:38 +0100] rev 22277
Fixed bug in mk_AbsP.
berghofe [Wed, 07 Feb 2007 17:59:40 +0100] rev 22276
Introduction and elimination rules for <= on predicates
are now declared properly.
berghofe [Wed, 07 Feb 2007 17:58:50 +0100] rev 22275
- Improved handling of monotonicity rules involving <=
- ind_cases: variables to be generalized can now be
specified using "for" keyword
berghofe [Wed, 07 Feb 2007 17:51:38 +0100] rev 22274
Adapted to changes in Finite_Set theory.
berghofe [Wed, 07 Feb 2007 17:46:03 +0100] rev 22273
Adapted to changes in Finite_Set theory.
berghofe [Wed, 07 Feb 2007 17:45:03 +0100] rev 22272
- Adapted to new inductive definition package
- More elegant proof of eta postponement theorem inspired
by Andreas Abel
berghofe [Wed, 07 Feb 2007 17:44:07 +0100] rev 22271
Adapted to new inductive definition package.
berghofe [Wed, 07 Feb 2007 17:41:11 +0100] rev 22270
Converted to predicate notation.
berghofe [Wed, 07 Feb 2007 17:39:49 +0100] rev 22269
Adapted to changes in List theory.
berghofe [Wed, 07 Feb 2007 17:37:59 +0100] rev 22268
- wfP has been moved to theory Wellfounded_Recursion
- Accessible part now works on predicates, hence accP is
no longer needed
berghofe [Wed, 07 Feb 2007 17:35:28 +0100] rev 22267
Adapted to changes in Transitive_Closure theory.
berghofe [Wed, 07 Feb 2007 17:34:43 +0100] rev 22266
Adapted to new inductive definition package.
berghofe [Wed, 07 Feb 2007 17:32:52 +0100] rev 22265
Adapted to changes in Finite_Set theory.
berghofe [Wed, 07 Feb 2007 17:30:53 +0100] rev 22264
Theorems for converting between wf and wfP are now declared
as hints.
berghofe [Wed, 07 Feb 2007 17:29:41 +0100] rev 22263
- Adapted to new inductive definition package
- Predicate version of wellfoundedness
berghofe [Wed, 07 Feb 2007 17:28:09 +0100] rev 22262
Adapted to new inductive definition package.
berghofe [Wed, 07 Feb 2007 17:26:49 +0100] rev 22261
Adapted to changes in Transitive_Closure theory.
berghofe [Wed, 07 Feb 2007 17:26:04 +0100] rev 22260
Added Predicate theory.
berghofe [Wed, 07 Feb 2007 17:25:39 +0100] rev 22259
New theory for converting between predicates and sets.
bulwahn [Wed, 07 Feb 2007 13:05:28 +0100] rev 22258
changes in lexicographic_order termination tactic
berghofe [Wed, 07 Feb 2007 12:08:48 +0100] rev 22257
"prove" function now instantiates relation variable in order
to avoid problems with higher-order unification. This allows
relations to be encoded as binary predicates.
berghofe [Wed, 07 Feb 2007 12:05:54 +0100] rev 22256
Made untabify function tail recursive.
wenzelm [Tue, 06 Feb 2007 19:32:32 +0100] rev 22255
tuned matches_subterm;
wenzelm [Tue, 06 Feb 2007 19:32:31 +0100] rev 22254
trace/debug: avoid eager string concatenation;
wenzelm [Tue, 06 Feb 2007 18:02:28 +0100] rev 22253
cc: removed option -lstdc++, which seems to be unnecessry, but causes problems on some platforms;
wenzelm [Tue, 06 Feb 2007 17:20:14 +0100] rev 22252
pervasive exception Option;
fixed use_file;
wenzelm [Tue, 06 Feb 2007 17:06:44 +0100] rev 22251
added has_kind/get_kind;
tuned;
urbanc [Tue, 06 Feb 2007 15:12:18 +0100] rev 22250
fixed two stupid bugs of SML to do with the value restriction and missing type
information in records
aspinall [Tue, 06 Feb 2007 12:54:55 +0100] rev 22249
askids/qualified_thms_of_thy: version which returns names in domain of get_thm
haftmann [Tue, 06 Feb 2007 11:40:53 +0100] rev 22248
added eta expansion to imperative monad bind
urbanc [Tue, 06 Feb 2007 00:53:15 +0100] rev 22247
corrected typo introduced by me
urbanc [Tue, 06 Feb 2007 00:43:23 +0100] rev 22246
now obsolete
urbanc [Tue, 06 Feb 2007 00:41:54 +0100] rev 22245
moved the infrastructure from the nominal_tags file to nominal_thmdecls
file, and adapted the code to conform with informal Isabelle programming
conventions
krauss [Mon, 05 Feb 2007 15:55:32 +0100] rev 22244
Exporting curried versions of tail recursive equations instead of internal ones
wenzelm [Mon, 05 Feb 2007 12:03:52 +0100] rev 22243
proper use of NameSpace.is_qualified (avoids compatibility issues of the SML B library);
wenzelm [Sun, 04 Feb 2007 22:02:22 +0100] rev 22242
removed non-modular comment;
wenzelm [Sun, 04 Feb 2007 22:02:21 +0100] rev 22241
interpretation: attempt to be more serious about name_morphism;
wenzelm [Sun, 04 Feb 2007 22:02:20 +0100] rev 22240
added full_naming;
wenzelm [Sun, 04 Feb 2007 22:02:19 +0100] rev 22239
tuned oracle interface;
simproc_setup: added identifier;
wenzelm [Sun, 04 Feb 2007 22:02:18 +0100] rev 22238
added print_strings;
wenzelm [Sun, 04 Feb 2007 22:02:17 +0100] rev 22237
old-fashioned abstype ctyp/cterm/thm prevents accidental equality tests;