Thu, 14 Oct 2010 09:28:05 -0700 huffman add type annotation to avoid warning
Wed, 13 Oct 2010 10:56:42 -0700 huffman cleaned up Fun_Cpo.thy; deprecated a few theorem names
Wed, 13 Oct 2010 10:27:26 -0700 huffman edit comments
Tue, 12 Oct 2010 09:32:21 -0700 huffman remove unneeded lemmas Lift_exhaust, Lift_cases
Tue, 12 Oct 2010 09:08:27 -0700 huffman move lemmas from Lift.thy to Cfun.thy
Tue, 12 Oct 2010 07:46:44 -0700 huffman cleaned up Adm.thy
Tue, 12 Oct 2010 06:20:05 -0700 huffman remove unneeded lemmas from Fun_Cpo.thy
Tue, 12 Oct 2010 05:48:32 -0700 huffman remove unused lemmas
Tue, 12 Oct 2010 05:48:15 -0700 huffman reformulate lemma cont2cont_lub and move to Cont.thy
Tue, 12 Oct 2010 05:25:21 -0700 huffman remove unused lemmas cont_fst_snd_D1, cont_fst_snd_D2
Mon, 11 Oct 2010 21:35:31 -0700 huffman new theorem names: fun_below_iff, fun_belowI, cfun_eq_iff, cfun_eqI, cfun_below_iff, cfun_belowI
Mon, 11 Oct 2010 16:24:44 -0700 huffman rename Ffun.thy to Fun_Cpo.thy
Mon, 11 Oct 2010 16:14:15 -0700 huffman remove unused constant 'directed'
Mon, 11 Oct 2010 09:54:04 -0700 huffman add HOLCF/Library/Defl_Bifinite.thy, which proves instance defl :: bifinite
Fri, 15 Oct 2010 17:21:37 +0100 paulson merged
Fri, 15 Oct 2010 17:21:07 +0100 paulson prevention of self-referential type environments
Fri, 15 Oct 2010 21:50:26 +0900 Cezary Kaliszyk FSet: definition changes propagated from Nominal and more use of 'descending' tactic
Fri, 15 Oct 2010 21:47:45 +0900 Cezary Kaliszyk FSet tuned
Fri, 15 Oct 2010 21:46:45 +0900 Cezary Kaliszyk FSet: give names to respectfulness theorems, rename list_all2_refl to avoid clash
Thu, 14 Oct 2010 12:40:14 +0200 krauss NEWS
Sun, 10 Oct 2010 22:50:25 +0200 krauss removed output syntax "'a ~=> 'b" for "'a => 'b option"
Wed, 13 Oct 2010 09:56:00 +0200 krauss reactivated
Tue, 12 Oct 2010 21:30:44 +0200 krauss slightly more robust proof
Mon, 11 Oct 2010 08:32:09 -0700 huffman renamed type and constant 'sfp' to 'defl'; replaced syntax SFP('a) with DEFL('a)
Mon, 11 Oct 2010 07:09:42 -0700 huffman merged
Sat, 09 Oct 2010 07:24:49 -0700 huffman move all bifinite class instances to Bifinite.thy
Fri, 08 Oct 2010 07:39:50 -0700 huffman rename class 'sfp' to 'bifinite'
Thu, 07 Oct 2010 13:54:43 -0700 huffman move stuff from Algebraic.thy to Bifinite.thy and elsewhere
Thu, 07 Oct 2010 13:33:06 -0700 huffman add lemma typedef_ideal_completion
Thu, 07 Oct 2010 13:22:13 -0700 huffman remove unused lemmas
Thu, 07 Oct 2010 13:19:45 -0700 huffman remove Infinite_Set from ROOT.ML
Thu, 07 Oct 2010 13:18:48 -0700 huffman remove some junk that made it in by accient
Mon, 11 Oct 2010 18:03:47 +0700 blanchet "setup" in theory
Mon, 11 Oct 2010 18:03:18 +0700 blanchet added "trace_meson" configuration option, replacing old-fashioned reference
Mon, 11 Oct 2010 18:02:14 +0700 blanchet added "trace_metis" configuration option, replacing old-fashioned references
Sun, 10 Oct 2010 23:16:24 +0200 krauss do not mention unqualified names, now that 'global' and 'local' are gone
Sun, 10 Oct 2010 16:34:20 +0200 nipkow simplified proof
Sun, 10 Oct 2010 18:42:13 +0700 blanchet avoid generating several formulas with the same name ("tfrees")
Wed, 06 Oct 2010 10:49:27 -0700 huffman major reorganization/simplification of HOLCF type classes:
Tue, 05 Oct 2010 17:53:00 -0700 Brian Huffman add lemma finite_deflation_intro
Tue, 05 Oct 2010 17:36:45 -0700 Brian Huffman add lemmas finite_deflation_imp_compact, cast_below_cast_iff
Tue, 05 Oct 2010 17:32:02 -0700 Brian Huffman move lemmas to Deflation.thy
Tue, 05 Oct 2010 17:07:57 -0700 Brian Huffman simplify proofs of powerdomain inequalities
Mon, 04 Oct 2010 06:58:37 -0700 huffman new lemmas about lub
Mon, 04 Oct 2010 06:45:57 -0700 huffman define is_ub predicate using bounded quantifier
Sat, 02 Oct 2010 17:50:33 -0700 huffman minimize theory imports
Fri, 01 Oct 2010 07:40:57 -0700 huffman added lemmas to List_Cpo.thy
Thu, 30 Sep 2010 19:42:12 -0700 huffman new_domain emits proper error message when a constructor argument type does not have sort 'rep'
Wed, 06 Oct 2010 17:56:41 +0200 blanchet move code from "Metis_Tactics" to "Metis_Reconstruct"
Wed, 06 Oct 2010 17:44:21 +0200 blanchet merged
Wed, 06 Oct 2010 17:44:07 +0200 blanchet qualify "Meson." and "Metis." constants so that the ML files can be reloaded later (e.g. for testing/development)
Wed, 06 Oct 2010 17:42:57 +0200 blanchet get rid of function that duplicates existing Pure functionality
Wed, 06 Oct 2010 17:38:06 +0200 blanchet remove needless fact
Wed, 06 Oct 2010 12:01:55 +0200 blanchet added a few FIXMEs
Tue, 05 Oct 2010 12:50:45 +0200 blanchet tuned comments
Tue, 05 Oct 2010 12:06:08 +0200 blanchet document latest changes to Meson/Metis/Sledgehammer
Tue, 05 Oct 2010 12:04:57 +0200 blanchet remove needless Metis facts
Tue, 05 Oct 2010 12:04:49 +0200 blanchet hide one more name
Tue, 05 Oct 2010 12:04:19 +0200 blanchet qualify names
Tue, 05 Oct 2010 11:45:10 +0200 blanchet hide uninteresting MESON/Metis constants and facts and remove "meson_" prefix to (now hidden) fact names
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip