Fri, 02 Mar 2007 15:43:17 +0100 haftmann new code theorems
Fri, 02 Mar 2007 15:43:16 +0100 haftmann syntax for "class attach const"
Fri, 02 Mar 2007 15:43:15 +0100 haftmann prefix of class interpretation not mandatory any longer
Fri, 02 Mar 2007 12:38:58 +0100 paulson Meson.is_fol_term now takes a theory as argument. Minor tidying.
Fri, 02 Mar 2007 12:37:34 +0100 paulson New code to store theorem names in a concise form rather than as fully-qualified.
Fri, 02 Mar 2007 12:35:20 +0100 paulson The first-order test now tests for the obscure case of a polymorphic constant like 1 being
Wed, 28 Feb 2007 22:05:46 +0100 wenzelm abbrev: be permissive after transformation;
Wed, 28 Feb 2007 22:05:44 +0100 wenzelm exported get_ss, map_ss;
Wed, 28 Feb 2007 22:05:43 +0100 wenzelm tuned;
Wed, 28 Feb 2007 22:05:43 +0100 wenzelm tuned ML setup;
Wed, 28 Feb 2007 22:05:41 +0100 wenzelm added @{const_name}, @{const_syntax};
Wed, 28 Feb 2007 16:35:00 +0100 krauss more cleanup
Wed, 28 Feb 2007 14:46:21 +0100 aspinall Add closeblock/openblock structure to proof-block commands
Wed, 28 Feb 2007 13:33:10 +0100 paulson Updated success string for Vampire.
Wed, 28 Feb 2007 12:51:46 +0100 paulson Now outputs metis calls
Wed, 28 Feb 2007 11:12:12 +0100 krauss added headers
Wed, 28 Feb 2007 10:36:10 +0100 krauss cleanup, fixing sml/nj related problems
Wed, 28 Feb 2007 00:22:26 +0100 wenzelm gensym: removed bits of dead code;
Tue, 27 Feb 2007 11:10:35 +0100 paulson gensym no longer includes ' or _ in names (trailing _ is bad)
Tue, 27 Feb 2007 00:33:49 +0100 wenzelm tuned document;
Tue, 27 Feb 2007 00:32:52 +0100 wenzelm \usepackage{amssymb};
Mon, 26 Feb 2007 23:18:30 +0100 wenzelm moved some non-kernel material to more_thm.ML;
Mon, 26 Feb 2007 23:18:29 +0100 wenzelm removed obsolete eq_set;
Mon, 26 Feb 2007 23:18:28 +0100 wenzelm Thm.internalK;
Mon, 26 Feb 2007 23:18:27 +0100 wenzelm Further operations on type thm, outside the inference kernel.
Mon, 26 Feb 2007 23:18:26 +0100 wenzelm added more_thm.ML;
Mon, 26 Feb 2007 23:18:24 +0100 wenzelm moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
Mon, 26 Feb 2007 21:34:16 +0100 krauss Added formalization of size-change principle (experimental).
Mon, 26 Feb 2007 20:14:52 +0100 wenzelm added theorems_of;
Mon, 26 Feb 2007 20:14:47 +0100 wenzelm removed obsolete theorem_space;
Mon, 26 Feb 2007 15:08:37 +0100 krauss Added lemma lfp_const: "lfp (%x. t) = t
Fri, 23 Feb 2007 08:39:28 +0100 haftmann exported serializer parsers
Fri, 23 Feb 2007 08:39:27 +0100 haftmann proper treatment of -> as type constructor
Fri, 23 Feb 2007 08:39:26 +0100 haftmann tuned
Fri, 23 Feb 2007 08:39:25 +0100 haftmann add_path for naming in proof contexts
Fri, 23 Feb 2007 08:39:24 +0100 haftmann locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
Fri, 23 Feb 2007 08:39:23 +0100 haftmann slightly tuned
Fri, 23 Feb 2007 08:39:22 +0100 haftmann slight cleanup
Fri, 23 Feb 2007 08:39:21 +0100 haftmann adjusted code lemmas
Fri, 23 Feb 2007 08:39:20 +0100 haftmann continued
Fri, 23 Feb 2007 08:39:19 +0100 haftmann dropped diagnostic switch
Thu, 22 Feb 2007 10:25:14 +0100 paulson Improved handling of situation when theorem in cache disagrees with theorem supplied: new clauses
Wed, 21 Feb 2007 13:51:12 +0100 krauss Fixed print translations for quantifiers a la "ALL x>=t. P x". These used
Wed, 21 Feb 2007 02:30:06 +0100 kleing prevent quadratic time removal of duplicates if filter list is empty (likely to have too many results)
Tue, 20 Feb 2007 00:53:18 +0100 kleing added missing \
Tue, 20 Feb 2007 00:23:58 +0100 kleing updated docs with new with_dups syntax for find_theorems
Tue, 20 Feb 2007 00:14:33 +0100 kleing Remove duplicates from printed theorems in find_theorems
Mon, 19 Feb 2007 16:44:08 +0100 schirmer more precise error message in parameter unification
Sat, 17 Feb 2007 18:01:22 +0100 aspinall Updated
Sat, 17 Feb 2007 18:00:59 +0100 aspinall Fix <pgipquit>. Remove unused pgmlatomsN. Make showid match askids. Use string functions for showid, avoiding printwrap kludge.
Sat, 17 Feb 2007 17:22:53 +0100 aspinall <idvalue>: add name attribute to allow unsolicited updates.
Sat, 17 Feb 2007 17:19:59 +0100 aspinall pretty_full_theory: expose in signature.
Sat, 17 Feb 2007 17:18:47 +0100 aspinall Clarify comment
Fri, 16 Feb 2007 22:46:03 +0100 wenzelm unified arity parser/arguments;
Fri, 16 Feb 2007 22:13:16 +0100 wenzelm ML text: informative Output.debug only;
Fri, 16 Feb 2007 22:13:15 +0100 wenzelm unified arity parser/arguments;
Fri, 16 Feb 2007 19:19:19 +0100 berghofe Replaced "raise RecError" by "primrec_err" in function
Fri, 16 Feb 2007 11:01:16 +0100 schirmer added example for print-mode Axiom
Fri, 16 Feb 2007 11:00:47 +0100 schirmer added print-mode Axiom to print theorems without premises with a rule on top.
Fri, 16 Feb 2007 09:04:23 +0100 krauss updated Makefile
Thu, 15 Feb 2007 18:18:21 +0100 narboux start adding the attribute eqvt to some lemmas of the nominal library
Thu, 15 Feb 2007 17:35:19 +0100 krauss changed termination goal to use object quantifier
Thu, 15 Feb 2007 12:14:34 +0100 krauss added congruence rule for function composition
Thu, 15 Feb 2007 12:02:11 +0100 krauss beta_eta_contract specification befor processing. These normal forms avoid unpleasant surprises later on.
Wed, 14 Feb 2007 10:07:17 +0100 haftmann continued
Wed, 14 Feb 2007 10:06:17 +0100 haftmann class package now using Locale.interpretation_i
Wed, 14 Feb 2007 10:06:16 +0100 haftmann clarified explanation
Wed, 14 Feb 2007 10:06:15 +0100 haftmann cleanup
Wed, 14 Feb 2007 10:06:14 +0100 haftmann simpliefied instance statement
Wed, 14 Feb 2007 10:06:13 +0100 haftmann continued class tutorial
Wed, 14 Feb 2007 10:06:12 +0100 haftmann added class "preorder"
Tue, 13 Feb 2007 18:26:48 +0100 berghofe Added nominal_inductive keyword.
Tue, 13 Feb 2007 18:19:25 +0100 berghofe Added new file Nominal/nominal_inductive.ML
Tue, 13 Feb 2007 18:18:45 +0100 berghofe First steps towards strengthening of induction rules for
Tue, 13 Feb 2007 18:17:28 +0100 berghofe Added new file nominal_inductive.ML
Tue, 13 Feb 2007 18:16:50 +0100 berghofe Curried and exported mk_perm.
Tue, 13 Feb 2007 16:37:14 +0100 paulson COMP now performs a distinctness check on the multiple results before failing
Tue, 13 Feb 2007 10:09:21 +0100 bulwahn improved lexicographic order termination tactic
Sat, 10 Feb 2007 17:06:40 +0100 haftmann added OCaml example
Sat, 10 Feb 2007 16:43:23 +0100 paulson Completing the bug fix from the previous update: the result of unifying type
Sat, 10 Feb 2007 09:26:26 +0100 haftmann changed representation of constants; consistent name handling
Sat, 10 Feb 2007 09:26:25 +0100 haftmann changed representation of constants
Sat, 10 Feb 2007 09:26:24 +0100 haftmann tuned
Sat, 10 Feb 2007 09:26:23 +0100 haftmann new Isar command print_codesetup
Sat, 10 Feb 2007 09:26:22 +0100 haftmann added experimental class target
Sat, 10 Feb 2007 09:26:20 +0100 haftmann added class target stub
Sat, 10 Feb 2007 09:26:19 +0100 haftmann internal interfaces for interpretation and interpret
Sat, 10 Feb 2007 09:26:18 +0100 haftmann moved commands of class package here
Sat, 10 Feb 2007 09:26:17 +0100 haftmann added class package to Isar bootstrap
Sat, 10 Feb 2007 09:26:16 +0100 haftmann splut up code generation in two parts
Sat, 10 Feb 2007 09:26:15 +0100 haftmann canonical interface for attributes
Sat, 10 Feb 2007 09:26:14 +0100 haftmann changed name of interpretation linorder to order
Sat, 10 Feb 2007 09:26:12 +0100 haftmann adjusted to changes in class package
Sat, 10 Feb 2007 09:26:11 +0100 haftmann added outline for Isabelle library description
Sat, 10 Feb 2007 09:26:10 +0100 haftmann adjusted to new code generator Isar commands and changes in implementation
Sat, 10 Feb 2007 09:26:09 +0100 haftmann adjusted to new code generator Isar commands
Sat, 10 Feb 2007 09:26:08 +0100 haftmann added references for code generator tutorial
Sat, 10 Feb 2007 09:26:07 +0100 haftmann added antiquotation for exceptions
Sat, 10 Feb 2007 09:26:06 +0100 haftmann updated keywords
Thu, 08 Feb 2007 18:14:13 +0100 paulson cterm_instantiate was calling a type instantiation function that works only for matching,
Thu, 08 Feb 2007 17:22:22 +0100 urbanc added get-functions
Wed, 07 Feb 2007 18:12:58 +0100 berghofe Renamed member to memb to avoid confusion with member function
Wed, 07 Feb 2007 18:12:02 +0100 berghofe Adapted to changes in Finite_Set theory.
Wed, 07 Feb 2007 18:11:27 +0100 berghofe Adapted to new inductive definition package.
Wed, 07 Feb 2007 18:10:21 +0100 berghofe - Adapted to new inductive definition package
Wed, 07 Feb 2007 18:07:10 +0100 berghofe Added meta_spec to extraction_expand.
Wed, 07 Feb 2007 18:04:44 +0100 berghofe Added functions hhf_proof and un_hhf_proof.
Wed, 07 Feb 2007 18:03:18 +0100 berghofe Adapted to changes in Accessible_Part and Wellfounded_Recursion theories.
Wed, 07 Feb 2007 18:01:40 +0100 berghofe Added split_rule attribute.
Wed, 07 Feb 2007 18:00:38 +0100 berghofe Fixed bug in mk_AbsP.
Wed, 07 Feb 2007 17:59:40 +0100 berghofe Introduction and elimination rules for <= on predicates
Wed, 07 Feb 2007 17:58:50 +0100 berghofe - Improved handling of monotonicity rules involving <=
Wed, 07 Feb 2007 17:51:38 +0100 berghofe Adapted to changes in Finite_Set theory.
Wed, 07 Feb 2007 17:46:03 +0100 berghofe Adapted to changes in Finite_Set theory.
Wed, 07 Feb 2007 17:45:03 +0100 berghofe - Adapted to new inductive definition package
Wed, 07 Feb 2007 17:44:07 +0100 berghofe Adapted to new inductive definition package.
Wed, 07 Feb 2007 17:41:11 +0100 berghofe Converted to predicate notation.
Wed, 07 Feb 2007 17:39:49 +0100 berghofe Adapted to changes in List theory.
Wed, 07 Feb 2007 17:37:59 +0100 berghofe - wfP has been moved to theory Wellfounded_Recursion
Wed, 07 Feb 2007 17:35:28 +0100 berghofe Adapted to changes in Transitive_Closure theory.
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip