Tue, 18 Nov 2008 22:25:36 +0100 wenzelm fulfill_proof/thm_proof: commuted lazyness;
Tue, 18 Nov 2008 22:25:30 +0100 wenzelm fulfill_proof/thm_proof: commuted lazyness;
Tue, 18 Nov 2008 21:17:14 +0100 krauss removed lemmas called lemma1 and lemma2
Tue, 18 Nov 2008 18:25:59 +0100 wenzelm force_proofs after cumulative use_thys;
Tue, 18 Nov 2008 18:25:55 +0100 wenzelm signed_string_of_int for priorities;
Tue, 18 Nov 2008 18:25:52 +0100 wenzelm added force_proofs;
Tue, 18 Nov 2008 18:25:49 +0100 wenzelm added force_proofs (based on thms ever passed through enter_thms);
Tue, 18 Nov 2008 18:25:45 +0100 wenzelm tuned;
Tue, 18 Nov 2008 18:25:42 +0100 wenzelm eliminated rewrite_tac/fold_tac, which are not well-formed tactics due to change of main conclusion;
Tue, 18 Nov 2008 18:25:10 +0100 wenzelm moved table of standard Isabelle symbols to isar-ref manual;
Tue, 18 Nov 2008 18:22:49 +0100 wenzelm added isabelle-implementation manual;
Tue, 18 Nov 2008 13:19:13 +0100 wenzelm disabled threads -- as advertized;
Tue, 18 Nov 2008 11:26:59 +0100 wenzelm changes by Fabian Immler:
Tue, 18 Nov 2008 09:41:23 +0100 ballarin Code for switching to new locales.
Tue, 18 Nov 2008 09:40:44 +0100 ballarin add_thmss
Tue, 18 Nov 2008 09:40:06 +0100 ballarin Activate elements moved to element.ML.
Tue, 18 Nov 2008 00:11:06 +0100 wenzelm finish: force proofs;
Mon, 17 Nov 2008 23:34:35 +0100 wenzelm finish_proof: undefined promises may occur here;
Mon, 17 Nov 2008 23:17:13 +0100 wenzelm tuned promise/fullfill;
Mon, 17 Nov 2008 23:17:11 +0100 wenzelm unified treatment of PAxm/Oracle/Promise in basic proof term operations;
Mon, 17 Nov 2008 21:36:48 +0100 wenzelm removed Induct/Mutil.thy -- the file has been moved to AFP;
Mon, 17 Nov 2008 21:28:46 +0100 wenzelm simplified thm_deps -- no need to build a graph datastructure;
Mon, 17 Nov 2008 21:13:48 +0100 wenzelm removed Induct/Mutil.thy -- the file has been moved to AFP;
Mon, 17 Nov 2008 17:25:02 +0100 nipkow -> AFP
Mon, 17 Nov 2008 17:00:55 +0100 haftmann tuned unfold_locales invocation
Mon, 17 Nov 2008 17:00:27 +0100 haftmann explicit name morphism function for locale interpretation
Mon, 17 Nov 2008 17:00:26 +0100 haftmann Name.name_with_prefix (temporarily)
Mon, 17 Nov 2008 17:00:22 +0100 haftmann adjusted locale signature to *_cmd convention
Mon, 17 Nov 2008 17:00:21 +0100 haftmann whitespace tuning
Mon, 17 Nov 2008 14:03:39 +0100 ballarin Generic activation of locales.
Sun, 16 Nov 2008 22:12:44 +0100 wenzelm proof_body/pthm: removed redundant types field;
Sun, 16 Nov 2008 22:12:43 +0100 wenzelm put_name/thm_proof: promises are filled with fulfilled proofs;
Sun, 16 Nov 2008 22:12:41 +0100 wenzelm proof_body/pthm: removed redundant types field;
Sun, 16 Nov 2008 20:03:42 +0100 wenzelm clarified Thm.proof_body_of vs. Thm.proof_of;
Sun, 16 Nov 2008 18:19:27 +0100 berghofe - Corrected order of quantification over Frees.
Sun, 16 Nov 2008 18:18:45 +0100 berghofe Frees in PThms are now quantified in the order of their appearance in the
Sat, 15 Nov 2008 21:31:37 +0100 wenzelm adapted PThm and MinProof;
Sat, 15 Nov 2008 21:31:36 +0100 wenzelm retrieve thm deps from proof_body;
Sat, 15 Nov 2008 21:31:35 +0100 wenzelm retrieve thm deps from proof_body;
Sat, 15 Nov 2008 21:31:32 +0100 wenzelm adapted PThm;
Sat, 15 Nov 2008 21:31:30 +0100 wenzelm proof_of_term: removed obsolete disambiguisation table;
Sat, 15 Nov 2008 21:31:29 +0100 wenzelm rewrite_proof: simplified simprocs (no name required);
Sat, 15 Nov 2008 21:31:27 +0100 wenzelm Thm.proof_of returns proof_body;
Sat, 15 Nov 2008 21:31:25 +0100 wenzelm refined notion of derivation, consiting of promises and proof_body;
Sat, 15 Nov 2008 21:31:23 +0100 wenzelm reworked type proof: MinProof is vacous, added Promise, refined PThm (with serial);
Sat, 15 Nov 2008 21:31:21 +0100 wenzelm pretty_thm: oracle flag is always false for now (would require detailed check wrt. promises);
Sat, 15 Nov 2008 21:31:20 +0100 wenzelm ProofSyntax.proof_of_term: removed obsolete disambiguisation table;
Sat, 15 Nov 2008 21:31:19 +0100 wenzelm name_of_thm: Proofterm.fold_proof_atoms;
Sat, 15 Nov 2008 21:31:17 +0100 wenzelm Thm.proof_of returns proof_body;
Sat, 15 Nov 2008 21:31:15 +0100 wenzelm clean: added HOL-Main;
Sat, 15 Nov 2008 21:31:13 +0100 wenzelm rewrite_proof: simplified simprocs (no name required);
Sat, 15 Nov 2008 11:25:17 +0100 wenzelm multithreading support for polyml-5.2 actually disabled -- as advertized;
Fri, 14 Nov 2008 16:49:52 +0100 ballarin Initial part of locale reimplementation.
Fri, 14 Nov 2008 14:00:52 +0100 ballarin Made local_note_prefix public.
Fri, 14 Nov 2008 08:50:11 +0100 haftmann re-educated guess
Fri, 14 Nov 2008 08:50:10 +0100 haftmann namify and name_decl combinators
Fri, 14 Nov 2008 08:50:09 +0100 haftmann Name.is_nothing
Fri, 14 Nov 2008 08:50:08 +0100 haftmann lemmas about dom and minus / insert
Fri, 14 Nov 2008 08:50:07 +0100 haftmann added length_unique operation for code generation
Thu, 13 Nov 2008 22:45:12 +0100 wenzelm updated generated files;
Thu, 13 Nov 2008 22:44:40 +0100 wenzelm removed "includes" element (lost update?);
Thu, 13 Nov 2008 22:36:30 +0100 wenzelm updated generated files;
Thu, 13 Nov 2008 22:07:31 +0100 wenzelm added section "Explicit instantiation within a subgoal context";
Thu, 13 Nov 2008 22:06:36 +0100 wenzelm renamed "Rules" to "Object-level rules";
Thu, 13 Nov 2008 22:05:49 +0100 wenzelm more on basic tactics;
Thu, 13 Nov 2008 22:05:09 +0100 wenzelm basic ML reference for tactics;
Thu, 13 Nov 2008 22:04:19 +0100 wenzelm added section "Tactics";
Thu, 13 Nov 2008 22:03:26 +0100 wenzelm more contributors;
Thu, 13 Nov 2008 22:02:18 +0100 wenzelm separate section "Inspecting the syntax" for print_syntax;
Thu, 13 Nov 2008 22:01:30 +0100 wenzelm misc tuning of inner syntax;
Thu, 13 Nov 2008 22:00:39 +0100 wenzelm added inner lexical syntax, reusing outer one;
Thu, 13 Nov 2008 22:00:12 +0100 wenzelm misc tuning;
Thu, 13 Nov 2008 21:59:47 +0100 wenzelm tuned outer lexical syntax; fixed var/tvar: really need question marks here;
Thu, 13 Nov 2008 21:59:02 +0100 wenzelm more tuning of Pure grammer;
Thu, 13 Nov 2008 21:57:50 +0100 wenzelm updated and elaborated Pure grammer;
Thu, 13 Nov 2008 21:57:20 +0100 wenzelm added Pure grammer (from old ref manual);
Thu, 13 Nov 2008 21:56:49 +0100 wenzelm mixfix annotations: verbatim for special symbols;
Thu, 13 Nov 2008 21:56:23 +0100 wenzelm added section "The Pure grammar" (incomplete version, based on old ref manual);
Thu, 13 Nov 2008 21:54:51 +0100 wenzelm added section "Priority grammars" (variant from old ref manual);
Thu, 13 Nov 2008 21:53:54 +0100 wenzelm added section "Co-regularity of type classes and arities" (variant from old ref manual);
Thu, 13 Nov 2008 21:52:59 +0100 wenzelm minor tuning (according to old ref manual);
Thu, 13 Nov 2008 21:52:09 +0100 wenzelm misc tuning and rearrangement of section "Printing logical entities";
Thu, 13 Nov 2008 21:50:57 +0100 wenzelm misc tuning and rearrangement of section "Printing logical entities";
Thu, 13 Nov 2008 21:50:30 +0100 wenzelm fixed/tuned syntax for attribute "tagged";
Thu, 13 Nov 2008 21:49:46 +0100 wenzelm added pretty printing options (from old ref manual);
Thu, 13 Nov 2008 21:48:19 +0100 wenzelm separate chapter "Inner syntax --- the term language";
Thu, 13 Nov 2008 21:45:40 +0100 wenzelm updated/refined types of Isar language elements, removed special LaTeX macros;
Thu, 13 Nov 2008 21:43:46 +0100 wenzelm unified use of declaration environment with IsarImplementation;
Thu, 13 Nov 2008 21:41:04 +0100 wenzelm ignore ThyOutput.source flag;
Thu, 13 Nov 2008 21:40:30 +0100 wenzelm added bind_thm, bind_thms;
Thu, 13 Nov 2008 21:40:00 +0100 wenzelm tuned section "Incorporating ML code";
Thu, 13 Nov 2008 21:38:44 +0100 wenzelm tuned section "Oracles";
Thu, 13 Nov 2008 21:38:02 +0100 wenzelm tuned section arrangement;
Thu, 13 Nov 2008 21:37:18 +0100 wenzelm moved section "Proof method expressions" to proof chapter;
Thu, 13 Nov 2008 21:34:55 +0100 wenzelm more on mixfix annotations (updated material from old ref manual);
Thu, 13 Nov 2008 21:34:23 +0100 wenzelm tuned;
Thu, 13 Nov 2008 21:33:56 +0100 wenzelm moved section "Document preparation" to front;
Thu, 13 Nov 2008 21:33:15 +0100 wenzelm updated section "Markup via command tags";
Thu, 13 Nov 2008 21:32:36 +0100 wenzelm renamed "formal comments" to "document comments";
Thu, 13 Nov 2008 21:31:25 +0100 wenzelm renamed "formal comments" to "document comments";
Thu, 13 Nov 2008 21:30:41 +0100 wenzelm tuned "Markup commands";
Thu, 13 Nov 2008 21:29:19 +0100 wenzelm tuned intro of "Document preparation";
Thu, 13 Nov 2008 21:25:42 +0100 wenzelm reworked "Defining Theories";
Thu, 13 Nov 2008 17:56:36 +0100 haftmann removed Assert.thy
Thu, 13 Nov 2008 15:59:36 +0100 haftmann dropped superfluos eval_conv
Thu, 13 Nov 2008 15:59:33 +0100 haftmann moved assert to Heap_Monad.thy
Thu, 13 Nov 2008 15:58:38 +0100 haftmann simproc for let
Thu, 13 Nov 2008 15:58:37 +0100 haftmann improved handling of !!/==> for eval and normalization
Thu, 13 Nov 2008 14:19:10 +0100 haftmann proper name morphisms for locales
Thu, 13 Nov 2008 14:19:09 +0100 haftmann consider prefixes for name bindings of simprocs (a first approximation)
Thu, 13 Nov 2008 14:19:07 +0100 haftmann diagnostic output for name bindings
Thu, 13 Nov 2008 01:31:20 +0100 berghofe Some modifications in code for proving arities to make it work for datatype
Wed, 12 Nov 2008 17:23:22 +0100 krauss min_ext/max_ext lifting wellfounded relations on finite sets. Preserves wf
Mon, 10 Nov 2008 19:42:22 +0100 haftmann restruced naming code in anticipation of introduction of name morphisms
Mon, 10 Nov 2008 19:42:21 +0100 haftmann more verbose element printing
Mon, 10 Nov 2008 19:42:20 +0100 haftmann clarified comment
Mon, 10 Nov 2008 17:38:23 +0100 berghofe Added support for parametric datatypes.
Mon, 10 Nov 2008 17:37:25 +0100 berghofe Streamlined functions for accessing information about atoms.
Mon, 10 Nov 2008 17:34:26 +0100 berghofe Some more functions for accessing information about atoms.
Mon, 10 Nov 2008 14:36:49 +0100 ballarin Made doc compatible with the system.
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip