wenzelm [Thu, 22 Dec 2005 00:28:54 +0100] rev 18468
fixed has_internal;
added is_internal;
renamed imp_cong' to imp_cong_rule;
uniform versions of forall_conv, concl_conv, prems_conv, conjunction_conv;
wenzelm [Thu, 22 Dec 2005 00:28:53 +0100] rev 18467
Tactic.precise_conjunction_tac;
wenzelm [Thu, 22 Dec 2005 00:28:52 +0100] rev 18466
added locale meta_conjunction_syntax and various conjunction rules;
wenzelm [Thu, 22 Dec 2005 00:28:51 +0100] rev 18465
simplified setup: removed dest_concls, local_impI, conjI;
improved handling of simultaneous goals: split cases;
simplified treatment of mutual rules, which are now specified as a list
instead of object-level conjunction (cf. set/type/rule);
moved join_rules to RuleCases.mutual_rule;
wenzelm [Thu, 22 Dec 2005 00:28:49 +0100] rev 18464
induct_rulify;
wenzelm [Thu, 22 Dec 2005 00:28:47 +0100] rev 18463
actually produce projected rules;
*.inducts holds all projected rules;
wenzelm [Thu, 22 Dec 2005 00:28:46 +0100] rev 18462
*.inducts holds all projected rules;
wenzelm [Thu, 22 Dec 2005 00:28:44 +0100] rev 18461
tuned;
wenzelm [Thu, 22 Dec 2005 00:28:43 +0100] rev 18460
tuned induct proofs;
wenzelm [Thu, 22 Dec 2005 00:28:41 +0100] rev 18459
mutual induct with *.inducts;
wenzelm [Thu, 22 Dec 2005 00:28:39 +0100] rev 18458
wf_induct_rule: consumes 1;
wenzelm [Thu, 22 Dec 2005 00:28:36 +0100] rev 18457
structure ProjectRule;
updated auxiliary facts for induct method;
tuned proofs;
wenzelm [Thu, 22 Dec 2005 00:28:34 +0100] rev 18456
updated auxiliary facts for induct method;
haftmann [Wed, 21 Dec 2005 17:00:57 +0100] rev 18455
slight improvements
haftmann [Wed, 21 Dec 2005 15:19:16 +0100] rev 18454
slight improvements in name handling
haftmann [Wed, 21 Dec 2005 15:18:57 +0100] rev 18453
slight refinements
haftmann [Wed, 21 Dec 2005 15:18:36 +0100] rev 18452
added eq_ord
haftmann [Wed, 21 Dec 2005 15:18:17 +0100] rev 18451
slight clean ups
haftmann [Wed, 21 Dec 2005 13:25:20 +0100] rev 18450
discontinued unflat in favour of burrow and burrow_split
paulson [Wed, 21 Dec 2005 12:06:08 +0100] rev 18449
new hash table module in HOL/Too/s
paulson [Wed, 21 Dec 2005 12:05:47 +0100] rev 18448
modified suffix for [iff] attribute
paulson [Wed, 21 Dec 2005 12:02:57 +0100] rev 18447
removed or modified some instances of [iff]
wenzelm [Tue, 20 Dec 2005 22:06:00 +0100] rev 18446
tuned;
haftmann [Tue, 20 Dec 2005 09:02:41 +0100] rev 18445
added .cvsignore
haftmann [Tue, 20 Dec 2005 09:01:48 +0100] rev 18444
removed improper .cvsignore
haftmann [Tue, 20 Dec 2005 08:58:36 +0100] rev 18443
removed superfluos is_prefix functions
haftmann [Tue, 20 Dec 2005 08:38:43 +0100] rev 18442
resolved shadowing of Library.find_first
haftmann [Tue, 20 Dec 2005 08:38:10 +0100] rev 18441
removed infix prefix, introduces burrow
mengj [Tue, 20 Dec 2005 04:29:25 +0100] rev 18440
Literals in clauses are sorted now. Added functions for clause equivalence tests and hashing clauses to words.
mengj [Tue, 20 Dec 2005 04:27:46 +0100] rev 18439
Added functions for fol_type; also put some functions to the signature, used by ResHolClause.
urbanc [Mon, 19 Dec 2005 16:07:19 +0100] rev 18438
made the changes according to Florian's re-arranging of
tuples (everything up to 19th December).
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.