wenzelm [Sat, 04 Apr 1998 11:43:39 +0200] rev 4790
removed simple;
added fail, untag;
wenzelm [Sat, 04 Apr 1998 11:42:48 +0200] rev 4789
added triv_goal, rev_triv_goal (for Isar);
wenzelm [Sat, 04 Apr 1998 11:42:26 +0200] rev 4788
added Goal_def;
wenzelm [Sat, 04 Apr 1998 11:41:24 +0200] rev 4787
replaced thy_data by thy_setup;
wenzelm [Sat, 04 Apr 1998 11:41:00 +0200] rev 4786
added local_theory (for Isar);
added setup;
wenzelm [Sat, 04 Apr 1998 11:40:18 +0200] rev 4785
tuned trace msgs;
wenzelm [Fri, 03 Apr 1998 14:38:19 +0200] rev 4784
tuned names;
wenzelm [Fri, 03 Apr 1998 14:37:48 +0200] rev 4783
added get_tthm(s), store_tthms(s);
tuned;
wenzelm [Fri, 03 Apr 1998 14:36:20 +0200] rev 4782
tuned comments;
wenzelm [Fri, 03 Apr 1998 14:36:05 +0200] rev 4781
added attribute.ML;
wenzelm [Fri, 03 Apr 1998 14:35:39 +0200] rev 4780
Theorem tags and attributes.
paulson [Fri, 03 Apr 1998 13:32:42 +0200] rev 4779
UNITY
oheimb [Fri, 03 Apr 1998 13:30:49 +0200] rev 4778
repaired incompatibility with new SML version by eta-expansion
paulson [Fri, 03 Apr 1998 12:35:27 +0200] rev 4777
New target HOL-UNITY
paulson [Fri, 03 Apr 1998 12:34:33 +0200] rev 4776
New UNITY theory
paulson [Fri, 03 Apr 1998 11:22:51 +0200] rev 4775
Tidied proofs
paulson [Fri, 03 Apr 1998 11:20:41 +0200] rev 4774
Tidied proofs by getting rid of case_tac
oheimb [Fri, 03 Apr 1998 09:54:48 +0200] rev 4773
improved \tt appearance of many ASCII special symbols like #
isabelle theory file keywords now appear bold only when at begin of line
oheimb [Thu, 02 Apr 1998 17:19:02 +0200] rev 4772
split_all_tac now fails if there is nothing to split
split_all_tac has moved within claset() from usafe wrappers to safe wrappers
paulson [Thu, 02 Apr 1998 13:49:04 +0200] rev 4771
new theorems
paulson [Thu, 02 Apr 1998 13:48:48 +0200] rev 4770
changed if_bool_eq to if_bool_eq_conj
paulson [Thu, 02 Apr 1998 13:48:28 +0200] rev 4769
changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
paulson [Thu, 02 Apr 1998 13:47:03 +0200] rev 4768
New theorems card_Diff_le and card_insert_le; tidied
oheimb [Thu, 02 Apr 1998 12:45:47 +0200] rev 4767
introduced functions for updating the wrapper lists
merge_cs now uses merge_alists to merge wrapper lists, left cs has precedence!
oheimb [Thu, 02 Apr 1998 12:39:32 +0200] rev 4766
*** empty log message ***
oheimb [Mon, 30 Mar 1998 21:15:18 +0200] rev 4765
merge_cs now also merges safe and unsafe wrappers
oheimb [Mon, 30 Mar 1998 21:14:04 +0200] rev 4764
generalized appearance of trancl_into_rtrancl and r_into_trancl
added irrefl_tranclI, reflcl_trancl, trancl_reflcl, trancl_empty, rtrancl_empty
oheimb [Mon, 30 Mar 1998 21:09:46 +0200] rev 4763
adapted proof of finite_converse
oheimb [Mon, 30 Mar 1998 21:08:05 +0200] rev 4762
added wf_converse_trancl, adapted proof of wfrec
oheimb [Mon, 30 Mar 1998 21:06:09 +0200] rev 4761
added caveat
oheimb [Mon, 30 Mar 1998 21:05:25 +0200] rev 4760
added introduction and elimination rules for Univalent
oheimb [Mon, 30 Mar 1998 21:04:41 +0200] rev 4759
added Univalent_rel_pow
oheimb [Mon, 30 Mar 1998 21:04:13 +0200] rev 4758
removed superfluous use_thy
oheimb [Mon, 30 Mar 1998 21:03:14 +0200] rev 4757
removed superfluous translations
wenzelm [Tue, 24 Mar 1998 16:57:40 +0100] rev 4756
added try, single, many;
improved source: prompt;
oheimb [Tue, 24 Mar 1998 15:57:18 +0100] rev 4755
added cproj', and therefore extended prj
tried to fix polymorphism problem for take_defs. A full solution will require
significant changes.
oheimb [Tue, 24 Mar 1998 15:54:42 +0100] rev 4754
added cproj', and therefore extended prj
oheimb [Tue, 24 Mar 1998 15:53:47 +0100] rev 4753
improved checks
oheimb [Tue, 24 Mar 1998 15:51:37 +0100] rev 4752
added o2s
oheimb [Tue, 24 Mar 1998 15:49:32 +0100] rev 4751
added finite_acyclic_wf_converse: corrected 8bit chars
oheimb [Tue, 24 Mar 1998 15:46:34 +0100] rev 4750
added acyclicI
oheimb [Tue, 24 Mar 1998 15:46:08 +0100] rev 4749
added finite_acyclic_wf_converse
paulson [Mon, 23 Mar 1998 13:56:53 +0100] rev 4748
more thms
paulson [Mon, 16 Mar 1998 16:54:07 +0100] rev 4747
inverse -> converse
paulson [Mon, 16 Mar 1998 16:50:50 +0100] rev 4746
inverse -> converse
[It is standard terminology and also used in ZF]
paulson [Mon, 16 Mar 1998 16:47:57 +0100] rev 4745
re-ordered proofs
wenzelm [Fri, 13 Mar 1998 18:15:14 +0100] rev 4744
moved addsplits [expand_if] from HOL_basic_ss to HOL_ss;
oheimb [Thu, 12 Mar 1998 13:17:13 +0100] rev 4743
renamed not1_or to disj_not1, not2_or to disj_not2
oheimb [Thu, 12 Mar 1998 13:15:36 +0100] rev 4742
improved coding of delWrapper and delSWrapper
oheimb [Thu, 12 Mar 1998 13:13:19 +0100] rev 4741
addloop: added warning in case of overwriting a looper
nipkow [Thu, 12 Mar 1998 12:49:24 +0100] rev 4740
Made mutual simplification of prems a special case.
nipkow [Thu, 12 Mar 1998 12:48:49 +0100] rev 4739
Used merge_alists for loopers.
paulson [Thu, 12 Mar 1998 10:40:08 +0100] rev 4738
New, stronger rewrites
paulson [Thu, 12 Mar 1998 10:39:19 +0100] rev 4737
The theorem nat_neqE, and some tidying
paulson [Thu, 12 Mar 1998 10:37:58 +0100] rev 4736
New laws, mostly generalizing old "pred" ones
paulson [Wed, 11 Mar 1998 14:54:41 +0100] rev 4735
spy_analz_tac now handles individual conjuncts properly
paulson [Wed, 11 Mar 1998 11:05:30 +0100] rev 4734
new theorem
paulson [Wed, 11 Mar 1998 11:05:14 +0100] rev 4733
New theorem Image_eq_UN; deleted the silly vimage_inverse_Image
paulson [Wed, 11 Mar 1998 11:03:43 +0100] rev 4732
Arith.thy -> thy; proved a few new theorems
nipkow [Wed, 11 Mar 1998 10:17:16 +0100] rev 4731
New Asm_full_simp_tac shortens proof.