QuotMain.thy
Thu, 15 Oct 2009 11:55:52 +0200 Cezary Kaliszyk Cleaning the code, part 4
Thu, 15 Oct 2009 11:53:11 +0200 Christian Urban slightly improved tyRel
Thu, 15 Oct 2009 11:42:14 +0200 Cezary Kaliszyk Reordering the code, part 3
Thu, 15 Oct 2009 11:29:38 +0200 Cezary Kaliszyk Reordering the code, part 2.
Thu, 15 Oct 2009 11:25:25 +0200 Cezary Kaliszyk Reordering the code, part 1.
Thu, 15 Oct 2009 11:20:50 +0200 Cezary Kaliszyk Minor cleaning.
Thu, 15 Oct 2009 11:17:27 +0200 Cezary Kaliszyk The definition of Fold1
Thu, 15 Oct 2009 10:25:23 +0200 Cezary Kaliszyk A number of lemmas for REGULARIZE_TAC and regularizing card1.
Wed, 14 Oct 2009 18:13:16 +0200 Cezary Kaliszyk Proving the proper RepAbs version
Wed, 14 Oct 2009 16:23:49 +0200 Cezary Kaliszyk Forgot to save, second part of the commit
Wed, 14 Oct 2009 16:23:32 +0200 Cezary Kaliszyk Manually regularized list_induct2
Wed, 14 Oct 2009 12:05:39 +0200 Cezary Kaliszyk Fixed bug in regularise types. Now we can regularise list.induct.
Wed, 14 Oct 2009 11:23:55 +0200 Cezary Kaliszyk Function for checking recursively if lifting is needed
Wed, 14 Oct 2009 09:50:13 +0200 Cezary Kaliszyk Merge
Wed, 14 Oct 2009 09:47:16 +0200 Cezary Kaliszyk Proper handling of non-lifted quantifiers, testing type freezing.
Tue, 13 Oct 2009 22:22:15 +0200 Christian Urban slight simplification of atomize_thm
Tue, 13 Oct 2009 18:01:54 +0200 Cezary Kaliszyk atomize_thm and meta_quantify.
Tue, 13 Oct 2009 13:37:07 +0200 Cezary Kaliszyk Regularizing HOL all.
Tue, 13 Oct 2009 11:38:35 +0200 Cezary Kaliszyk ":" is used for being in a set, "IN" means something else...
Tue, 13 Oct 2009 11:03:55 +0200 Cezary Kaliszyk First (untested) version of regularize for abstractions.
Mon, 12 Oct 2009 23:39:14 +0200 Christian Urban slightly modified the parser
Mon, 12 Oct 2009 23:16:20 +0200 Christian Urban deleted diagnostic code
Mon, 12 Oct 2009 23:06:14 +0200 Christian Urban added quotient command (you need to update isar-keywords-prove.el)
Mon, 12 Oct 2009 16:31:29 +0200 Cezary Kaliszyk Bounded quantifier
Mon, 12 Oct 2009 15:47:27 +0200 Cezary Kaliszyk The tyREL function.
Mon, 12 Oct 2009 14:30:50 +0200 Christian Urban started some strange functions
Mon, 12 Oct 2009 13:58:31 +0200 Cezary Kaliszyk Further with the manual proof
Fri, 09 Oct 2009 17:05:45 +0200 Cezary Kaliszyk Further experiments with proving induction manually
Fri, 09 Oct 2009 15:03:43 +0200 Cezary Kaliszyk Testing if I can prove the regularized version of induction manually
Thu, 08 Oct 2009 14:27:50 +0200 Christian Urban exported parts of QuotMain into a separate ML-file
Tue, 06 Oct 2009 15:11:30 +0200 Christian Urban consistent usage of rty (for the raw, unquotient type); tuned a bit the Isar
Tue, 06 Oct 2009 11:56:23 +0200 Christian Urban simplified typedef_quot_type_tac (using MetaSimplifier.rewrite_rule instead of the simplifier)
Tue, 06 Oct 2009 11:41:35 +0200 Christian Urban renamed unlam_def to unabs_def (matching the function abs_def in drule.ML)
Tue, 06 Oct 2009 11:36:08 +0200 Christian Urban tuned; nothing serious
Tue, 06 Oct 2009 09:28:59 +0200 Christian Urban another improvement to unlam_def
Tue, 06 Oct 2009 02:02:51 +0200 Christian Urban one further improvement to unlam_def
Tue, 06 Oct 2009 01:50:13 +0200 Christian Urban simplified the unlam_def function
Mon, 05 Oct 2009 11:54:02 +0200 Christian Urban added an explicit syntax-argument to the function make_def (is needed if the user gives an syntax annotation for quotient types)
Mon, 05 Oct 2009 11:24:32 +0200 Christian Urban used prop_of to get the term of a theorem (replaces crep_thm)
Fri, 02 Oct 2009 11:10:21 +0200 Cezary Kaliszyk Merged
Fri, 02 Oct 2009 11:09:33 +0200 Cezary Kaliszyk First theorem with quantifiers. Learned how to use sledgehammer.
Thu, 01 Oct 2009 16:10:14 +0200 Christian Urban simplified the storage of the map-functions by using TheoryDataFun
Wed, 30 Sep 2009 16:57:09 +0200 Cezary Kaliszyk Just one atomize is enough for the currently lifted theorems. Properly lift 'all' and 'Ex'.
Tue, 29 Sep 2009 22:35:48 +0200 Christian Urban used new cong_tac
Tue, 29 Sep 2009 17:46:18 +0200 Cezary Kaliszyk First version of handling of the universal quantifier
Tue, 29 Sep 2009 15:58:14 +0200 Cezary Kaliszyk Handling abstraction correctly.
Tue, 29 Sep 2009 13:38:27 +0200 Cezary Kaliszyk second test
Tue, 29 Sep 2009 13:24:57 +0200 Cezary Kaliszyk Test line
Tue, 29 Sep 2009 11:55:37 +0200 Cezary Kaliszyk Partially fix lifting of card_suc. The quantified variable still needs to be changed.
Tue, 29 Sep 2009 10:49:31 +0200 Cezary Kaliszyk Tested new build_goal and removed old one, eq_reflection is included in atomize, card_suc tests.
Tue, 29 Sep 2009 09:58:02 +0200 Cezary Kaliszyk Checked again with the version on my hard-drive backedup yesterday and fixed small whitespace issues.
Tue, 29 Sep 2009 09:26:22 +0200 Cezary Kaliszyk Merged
Mon, 28 Sep 2009 19:24:55 +0200 Christian Urban consistent state
Mon, 28 Sep 2009 19:22:28 +0200 Christian Urban some tuning of my code
Mon, 28 Sep 2009 19:15:19 +0200 Cezary Kaliszyk Cleanup
Mon, 28 Sep 2009 19:10:27 +0200 Cezary Kaliszyk Merged
Mon, 28 Sep 2009 18:59:04 +0200 Cezary Kaliszyk Cleaning the code with Makarius
Mon, 28 Sep 2009 15:37:38 +0200 Cezary Kaliszyk Instnatiation with a schematic variable
Mon, 28 Sep 2009 02:39:44 +0200 Christian Urban added ctxt as explicit argument to build_goal; tuned
Fri, 25 Sep 2009 19:26:18 +0200 Christian Urban slightly tuned the comment for unlam
Fri, 25 Sep 2009 17:08:50 +0200 Christian Urban fixed a bug in my code: function typedef_term constructs now now the correct term when the relation is called x
Fri, 25 Sep 2009 16:50:11 +0200 Christian Urban tuned slightly one proof
Fri, 25 Sep 2009 14:50:35 +0200 Cezary Kaliszyk A version of the tactic that exports variables correctly.
Fri, 25 Sep 2009 09:38:16 +0200 Cezary Kaliszyk Minor cleaning: whitespace, commas etc.
Thu, 24 Sep 2009 17:43:26 +0200 Cezary Kaliszyk Correctly handling abstractions while building goals
Thu, 24 Sep 2009 13:32:52 +0200 Cezary Kaliszyk Minor cleanup
Thu, 24 Sep 2009 11:38:20 +0200 Cezary Kaliszyk Found the source for the exception and added a handle for it.
Thu, 24 Sep 2009 09:09:46 +0200 Cezary Kaliszyk Make the tactic use Trueprop_cong and atomize.
Wed, 23 Sep 2009 16:57:56 +0200 Cezary Kaliszyk Proper code for getting the prop out of the theorem.
Wed, 23 Sep 2009 16:44:56 +0200 Cezary Kaliszyk Using "atomize" the versions with arbitrary Trueprops can be proven.
Tue, 22 Sep 2009 17:39:52 +0200 Cezary Kaliszyk Proper definition of CARD and some properties of it.
Tue, 22 Sep 2009 09:42:27 +0200 Christian Urban some comments
Mon, 21 Sep 2009 18:18:29 +0200 Christian Urban merged
Mon, 21 Sep 2009 18:18:01 +0200 Christian Urban slight tuning
Mon, 21 Sep 2009 16:45:44 +0200 Cezary Kaliszyk The tactic with REPEAT, CHANGED and a proper simpset.
Mon, 21 Sep 2009 10:53:01 +0200 Cezary Kaliszyk Merged with my changes from the morning:
Sun, 20 Sep 2009 05:48:49 +0100 Ning some more beautification
Sun, 20 Sep 2009 05:18:36 +0100 Ning beautification of some proofs
Fri, 18 Sep 2009 17:30:33 +0200 Cezary Kaliszyk Added more useful quotient facts.
Fri, 18 Sep 2009 13:44:06 +0200 Cezary Kaliszyk Testing the tactic further.
Thu, 17 Sep 2009 16:55:11 +0200 Cezary Kaliszyk The tactic still only for fset
Thu, 17 Sep 2009 12:06:06 +0200 Cezary Kaliszyk Infrastructure for the tactic
Wed, 16 Sep 2009 11:50:41 +0200 Cezary Kaliszyk More naming/binding suggestions from Makarius
Tue, 15 Sep 2009 11:31:35 +0200 Cezary Kaliszyk Code cleanup
Tue, 15 Sep 2009 10:00:34 +0200 Cezary Kaliszyk Cleaning the code
Tue, 15 Sep 2009 09:59:56 +0200 Cezary Kaliszyk Generalized interpretation, works for all examples.
Fri, 28 Aug 2009 17:12:19 +0200 Cezary Kaliszyk Fixes after suggestions from Makarius:
Fri, 28 Aug 2009 10:01:25 +0200 Cezary Kaliszyk More examples.
Thu, 27 Aug 2009 09:04:39 +0200 Cezary Kaliszyk Use metavariables in the 'non-lambda' definitions
Wed, 26 Aug 2009 11:31:55 +0200 Cezary Kaliszyk Make both kinds of definitions.
Tue, 25 Aug 2009 17:37:50 +0200 Cezary Kaliszyk Changed to the use of "modern interface"
Tue, 25 Aug 2009 14:37:11 +0200 Cezary Kaliszyk Initial version of the function that builds goals.
Tue, 25 Aug 2009 10:35:28 +0200 Cezary Kaliszyk - Build an interpretation for fset from ML level and use it
Tue, 25 Aug 2009 00:30:23 +0200 Christian Urban added the prove command
Fri, 21 Aug 2009 13:56:20 +0200 Cezary Kaliszyk Fixed
Fri, 21 Aug 2009 13:36:58 +0200 Christian Urban tuned
Thu, 20 Aug 2009 14:44:29 +0200 cek UNION - Append theorem
Thu, 20 Aug 2009 10:31:44 +0200 Christian Urban update
Tue, 18 Aug 2009 14:04:51 +0200 Christian Urban updated slightly
Tue, 11 Aug 2009 12:29:15 +0200 Christian Urban initial commit
less more (0) tip