urbanc [Mon, 19 Dec 2005 15:29:51 +0100] rev 18437
added proofs to show that every atom-kind combination
is in the respective finite-support class (now have to
adjust the files according to Florian's changes)
urbanc [Mon, 19 Dec 2005 12:58:15 +0100] rev 18436
added thms to perm_compose (so far only composition
theorems were included where the type of the permutation
was equal)
urbanc [Mon, 19 Dec 2005 12:09:56 +0100] rev 18435
tuned one comment
urbanc [Mon, 19 Dec 2005 12:08:16 +0100] rev 18434
fixed a bug that occured when more than one atom-type
is declared.
nipkow [Mon, 19 Dec 2005 09:19:08 +0100] rev 18433
fixed proof
urbanc [Sun, 18 Dec 2005 20:10:15 +0100] rev 18432
more cleaning up - this time of the cp-instance
proofs
urbanc [Sun, 18 Dec 2005 14:36:42 +0100] rev 18431
improved the finite-support proof
added finite support proof for options (I am
surprised that one does not need more fs-proofs;
at the moment only lists, products, units and
atoms are shown to be finitely supported (of
course also every nominal datatype is finitely
supported))
deleted pt_bool_inst - not necessary because discrete
types are treated separately in nominal_atoms
urbanc [Sun, 18 Dec 2005 13:38:06 +0100] rev 18430
improved the code for showing that a type is
in the pt-axclass (I try to slowly overcome
my incompetence with such ML-code).
wenzelm [Sat, 17 Dec 2005 01:58:41 +0100] rev 18429
simp del: empty_Collect_eq;
wenzelm [Sat, 17 Dec 2005 01:00:40 +0100] rev 18428
sort_distinct;
wenzelm [Sat, 17 Dec 2005 01:00:38 +0100] rev 18427
added sort_distinct;
removed obsolete unique_strings;
urbanc [Fri, 16 Dec 2005 18:22:58 +0100] rev 18426
added container-lemma fresh_eqvt
(definition: container-lemma contains all instantiations
of a lemma from the general theory)
urbanc [Fri, 16 Dec 2005 18:20:59 +0100] rev 18425
I think the earlier version was completely broken
(not sure about this one)
urbanc [Fri, 16 Dec 2005 18:20:03 +0100] rev 18424
tuned more proofs
nipkow [Fri, 16 Dec 2005 16:59:32 +0100] rev 18423
new lemmas
haftmann [Fri, 16 Dec 2005 16:00:58 +0100] rev 18422
re-arranged tuples (theory * 'a) to ('a * theory) in Pure
haftmann [Fri, 16 Dec 2005 15:52:05 +0100] rev 18421
re-arranged tuples (theory * 'a) to ('a * theory) in Pure
paulson [Fri, 16 Dec 2005 12:15:54 +0100] rev 18420
hashing to eliminate the output of duplicate clauses
paulson [Fri, 16 Dec 2005 11:51:24 +0100] rev 18419
hash tables from SML/NJ
haftmann [Fri, 16 Dec 2005 09:00:11 +0100] rev 18418
re-arranged tuples (theory * 'a) to ('a * theory) in Pure
urbanc [Thu, 15 Dec 2005 21:51:31 +0100] rev 18417
there was a small error in the last commit - fixed now
urbanc [Thu, 15 Dec 2005 21:49:14 +0100] rev 18416
tuned more proof and added in-file documentation
wenzelm [Thu, 15 Dec 2005 19:42:03 +0100] rev 18415
improved proofs;
wenzelm [Thu, 15 Dec 2005 19:42:02 +0100] rev 18414
acc_induct: proper tags;
wenzelm [Thu, 15 Dec 2005 19:42:00 +0100] rev 18413
removed obsolete/unused setup_induction;
urbanc [Thu, 15 Dec 2005 18:13:40 +0100] rev 18412
tuned the proof of transitivity/narrowing
paulson [Thu, 15 Dec 2005 15:26:37 +0100] rev 18411
No axiom, arity or classrel clauses contain HOL.type. Negative occurrences are
deleted; any positive occurrence of HOL.type kills the entire clause.
urbanc [Thu, 15 Dec 2005 11:53:38 +0100] rev 18410
made further tunings
mengj [Thu, 15 Dec 2005 05:47:26 +0100] rev 18409
Added functions to test equivalence between clauses.
webertj [Wed, 14 Dec 2005 22:05:22 +0100] rev 18408
ex/Sudoku.thy
paulson [Wed, 14 Dec 2005 18:01:50 +0100] rev 18407
deleted redundant (looping!) simprule
paulson [Wed, 14 Dec 2005 16:14:41 +0100] rev 18406
modified example for new clauses
paulson [Wed, 14 Dec 2005 16:14:26 +0100] rev 18405
removal of some redundancies (e.g. one-point-rules) in clause production
paulson [Wed, 14 Dec 2005 16:13:09 +0100] rev 18404
removed unused function repeat_RS
mengj [Wed, 14 Dec 2005 06:19:33 +0100] rev 18403
Changed literals' ordering and the functions for sorting literals.
mengj [Wed, 14 Dec 2005 01:40:43 +0100] rev 18402
1. changed fol_type, it's not a string type anymore.
2. sort literals in clauses.
mengj [Wed, 14 Dec 2005 01:39:41 +0100] rev 18401
changed ATP input files' names and location.
wenzelm [Tue, 13 Dec 2005 19:32:36 +0100] rev 18400
Potentially infinite lists as greatest fixed-point.
wenzelm [Tue, 13 Dec 2005 19:32:06 +0100] rev 18399
Provers/induct: coinduct;
HOL/Library: theory Coinductive_List;
wenzelm [Tue, 13 Dec 2005 19:32:05 +0100] rev 18398
tuned proofs;
wenzelm [Tue, 13 Dec 2005 19:32:04 +0100] rev 18397
added HOL/Library/Coinductive_List.thy;
urbanc [Tue, 13 Dec 2005 18:11:21 +0100] rev 18396
added a fresh_left lemma that contains all instantiation
for the various atom-types.
urbanc [Tue, 13 Dec 2005 16:30:50 +0100] rev 18395
initial commit (not to be seen by the public)
chaieb [Tue, 13 Dec 2005 16:25:10 +0100] rev 18394
simpset for computation in raw_arith_tac added just as comment, nothing changed!
chaieb [Tue, 13 Dec 2005 16:24:12 +0100] rev 18393
deals with Suc in mod expressions
wenzelm [Tue, 13 Dec 2005 15:46:41 +0100] rev 18392
Poplog/pml provides a proper print function already!
paulson [Tue, 13 Dec 2005 15:34:21 +0100] rev 18391
meson no longer does these examples
paulson [Tue, 13 Dec 2005 15:34:02 +0100] rev 18390
now generates the name "append"
paulson [Tue, 13 Dec 2005 15:27:43 +0100] rev 18389
removal of functional reflexivity axioms
berghofe [Tue, 13 Dec 2005 10:39:32 +0100] rev 18388
list_of_indset now also generates code for set type.
haftmann [Mon, 12 Dec 2005 17:24:06 +0100] rev 18387
added generic name mangler
haftmann [Mon, 12 Dec 2005 15:37:35 +0100] rev 18386
improvement in eq handling
haftmann [Mon, 12 Dec 2005 15:37:05 +0100] rev 18385
improvements in class and eq handling
haftmann [Mon, 12 Dec 2005 15:36:46 +0100] rev 18384
added dummy 'print' to non-polyml systems
urbanc [Sun, 11 Dec 2005 11:57:01 +0100] rev 18383
ISAR-fied some proofs
urbanc [Sun, 11 Dec 2005 01:21:26 +0100] rev 18382
completed the sn proof and changed the manual
accordingly
urbanc [Sat, 10 Dec 2005 00:11:35 +0100] rev 18381
changed the types in accordance with Florian's changes
haftmann [Fri, 09 Dec 2005 15:25:52 +0100] rev 18380
substantial improvements for class code generation
haftmann [Fri, 09 Dec 2005 15:25:29 +0100] rev 18379
improved extraction interface
urbanc [Fri, 09 Dec 2005 12:38:49 +0100] rev 18378
tuned
haftmann [Fri, 09 Dec 2005 09:06:45 +0100] rev 18377
oriented result pairs in PureThy
wenzelm [Thu, 08 Dec 2005 20:16:17 +0100] rev 18376
tuned;
wenzelm [Thu, 08 Dec 2005 20:16:10 +0100] rev 18375
removed Syntax.deskolem;
wenzelm [Thu, 08 Dec 2005 20:16:04 +0100] rev 18374
swap: no longer pervasive;
wenzelm [Thu, 08 Dec 2005 20:15:57 +0100] rev 18373
replaced swap by contrapos_np;
wenzelm [Thu, 08 Dec 2005 20:15:50 +0100] rev 18372
tuned proofs;
wenzelm [Thu, 08 Dec 2005 20:15:41 +0100] rev 18371
Cla.swap;
wenzelm [Thu, 08 Dec 2005 20:15:34 +0100] rev 18370
removed hint for Classical.swap, which is not really user-level anyway;
wenzelm [Thu, 08 Dec 2005 12:50:04 +0100] rev 18369
tuned sources and proofs
wenzelm [Thu, 08 Dec 2005 12:50:03 +0100] rev 18368
Classical.swap;
wenzelm [Thu, 08 Dec 2005 12:50:02 +0100] rev 18367
* HOL: Theorem 'swap' is no longer bound at the ML top-level.
berghofe [Thu, 08 Dec 2005 10:17:21 +0100] rev 18366
Adapted to new type of PureThy.add_defs_i.
wenzelm [Wed, 07 Dec 2005 16:47:04 +0100] rev 18365
replaced swap by Classical.swap;
wenzelm [Wed, 07 Dec 2005 15:23:22 +0100] rev 18364
avoid unportable tail;
urbanc [Wed, 07 Dec 2005 12:33:38 +0100] rev 18363
tuned
haftmann [Tue, 06 Dec 2005 17:26:26 +0100] rev 18362
removed thms 'swap' and 'nth_map' from ML toplevel
haftmann [Tue, 06 Dec 2005 17:11:40 +0100] rev 18361
improved serialization of classes to haskell
haftmann [Tue, 06 Dec 2005 16:07:25 +0100] rev 18360
improved class handling
haftmann [Tue, 06 Dec 2005 16:07:10 +0100] rev 18359
added 'dig' combinator
haftmann [Tue, 06 Dec 2005 09:04:09 +0100] rev 18358
re-oriented some result tuples in PureThy
mengj [Tue, 06 Dec 2005 06:22:14 +0100] rev 18357
Added more functions for new type embedding of HOL clauses.
mengj [Tue, 06 Dec 2005 06:21:07 +0100] rev 18356
Added new type embedding methods for translating HOL clauses.
urbanc [Mon, 05 Dec 2005 18:19:49 +0100] rev 18355
added code to say that discrete types (nat, bool, char)
are instances of cp_*_*.
urbanc [Mon, 05 Dec 2005 17:02:20 +0100] rev 18354
tuned
urbanc [Mon, 05 Dec 2005 15:55:19 +0100] rev 18353
transitivity should be now in a reasonable state. But
Markus has to have a look at some of the advanced features.
urbanc [Mon, 05 Dec 2005 10:33:30 +0100] rev 18352
tuned
urbanc [Mon, 05 Dec 2005 10:32:37 +0100] rev 18351
ISAR-fied two proofs
berghofe [Mon, 05 Dec 2005 00:39:18 +0100] rev 18350
Adapted to new type of store_thmss(_atts).
berghofe [Mon, 05 Dec 2005 00:38:07 +0100] rev 18349
Added store_thmss_atts to signature again.
urbanc [Sun, 04 Dec 2005 12:40:39 +0100] rev 18348
tuned
urbanc [Sun, 04 Dec 2005 12:25:57 +0100] rev 18347
tuned
urbanc [Sun, 04 Dec 2005 12:14:40 +0100] rev 18346
tuned
urbanc [Sun, 04 Dec 2005 12:14:27 +0100] rev 18345
added an Isar-proof for the abs_ALL lemma
urbanc [Sun, 04 Dec 2005 12:14:03 +0100] rev 18344
tuning
wenzelm [Fri, 02 Dec 2005 22:57:36 +0100] rev 18343
defines: beta/eta contract lhs;
replaced type_syntax by mixfix_type, which handles binders as well;
wenzelm [Fri, 02 Dec 2005 22:54:52 +0100] rev 18342
asts_to_terms: builtin free_fixed translation makes local binders work properly;