Tue, 10 Apr 2007 08:19:20 +0200 added example for definitions in local contexts
krauss [Tue, 10 Apr 2007 08:19:20 +0200] rev 22618
added example for definitions in local contexts
Tue, 10 Apr 2007 08:09:28 +0200 removed obsolete workaround
krauss [Tue, 10 Apr 2007 08:09:28 +0200] rev 22617
removed obsolete workaround
Mon, 09 Apr 2007 21:28:24 +0200 generalized type of lemma setsum_product
huffman [Mon, 09 Apr 2007 21:28:24 +0200] rev 22616
generalized type of lemma setsum_product
Mon, 09 Apr 2007 04:51:28 +0200 new standard proofs of some LIMSEQ lemmas
huffman [Mon, 09 Apr 2007 04:51:28 +0200] rev 22615
new standard proofs of some LIMSEQ lemmas
Sun, 08 Apr 2007 18:35:19 +0200 rearranged sections
huffman [Sun, 08 Apr 2007 18:35:19 +0200] rev 22614
rearranged sections
Sun, 08 Apr 2007 17:54:52 +0200 remove redundant lemmas
huffman [Sun, 08 Apr 2007 17:54:52 +0200] rev 22613
remove redundant lemmas
Sat, 07 Apr 2007 18:54:30 +0200 removed obsolete workarounds
krauss [Sat, 07 Apr 2007 18:54:30 +0200] rev 22612
removed obsolete workarounds
Sat, 07 Apr 2007 12:40:32 +0200 deleted remaining instances of swap_simp_a and swap_simp_b (obsolete now)
urbanc [Sat, 07 Apr 2007 12:40:32 +0200] rev 22611
deleted remaining instances of swap_simp_a and swap_simp_b (obsolete now)
Sat, 07 Apr 2007 11:36:35 +0200 tuned slightly the previous commit
urbanc [Sat, 07 Apr 2007 11:36:35 +0200] rev 22610
tuned slightly the previous commit
Sat, 07 Apr 2007 11:05:25 +0200 perm_simp can now simplify using the rules (a,b) o a = b and (a,b) o b = a
narboux [Sat, 07 Apr 2007 11:05:25 +0200] rev 22609
perm_simp can now simplify using the rules (a,b) o a = b and (a,b) o b = a
Fri, 06 Apr 2007 01:26:30 +0200 add new standard proofs for limits of sequences
huffman [Fri, 06 Apr 2007 01:26:30 +0200] rev 22608
add new standard proofs for limits of sequences
Thu, 05 Apr 2007 14:56:54 +0200 Replaced add_inductive_i by add_inductive_global.
berghofe [Thu, 05 Apr 2007 14:56:54 +0200] rev 22607
Replaced add_inductive_i by add_inductive_global.
Thu, 05 Apr 2007 14:56:10 +0200 - Tried to make name_of_thm more robust against changes of the
berghofe [Thu, 05 Apr 2007 14:56:10 +0200] rev 22606
- Tried to make name_of_thm more robust against changes of the structure of proofs. - Now uses add_inductive_global rather than add_inductive_i for the definition of the realizability predicate.
Thu, 05 Apr 2007 14:51:28 +0200 - Removed occurrences of ProofContext.export in add_ind_def that
berghofe [Thu, 05 Apr 2007 14:51:28 +0200] rev 22605
- Removed occurrences of ProofContext.export in add_ind_def that caused theorems to end up in the wrong context - Explicit parameters are now generalized in theorems returned by add_inductive(_i)
Thu, 05 Apr 2007 00:30:32 +0200 thy_deps: sort Context.thy_ord;
wenzelm [Thu, 05 Apr 2007 00:30:32 +0200] rev 22604
thy_deps: sort Context.thy_ord;
Thu, 05 Apr 2007 00:30:31 +0200 added thy_ord -- order of creation;
wenzelm [Thu, 05 Apr 2007 00:30:31 +0200] rev 22603
added thy_ord -- order of creation; ancestors: back to traditional ad-hoc order (avoid occasional problems with get_thm);
Wed, 04 Apr 2007 23:29:42 +0200 simplified thy_deps using Theory.ancestors_of (in order of creation);
wenzelm [Wed, 04 Apr 2007 23:29:42 +0200] rev 22602
simplified thy_deps using Theory.ancestors_of (in order of creation);
Wed, 04 Apr 2007 23:29:41 +0200 renamed Variable.importT to importT_thms;
wenzelm [Wed, 04 Apr 2007 23:29:41 +0200] rev 22601
renamed Variable.importT to importT_thms;
Wed, 04 Apr 2007 23:29:40 +0200 removed unused dep_graph;
wenzelm [Wed, 04 Apr 2007 23:29:40 +0200] rev 22600
removed unused dep_graph;
Wed, 04 Apr 2007 23:29:39 +0200 theory: maintain ancestors in order of creation;
wenzelm [Wed, 04 Apr 2007 23:29:39 +0200] rev 22599
theory: maintain ancestors in order of creation;
Wed, 04 Apr 2007 23:29:38 +0200 rep_thm/cterm/ctyp: removed obsolete sign field;
wenzelm [Wed, 04 Apr 2007 23:29:38 +0200] rev 22598
rep_thm/cterm/ctyp: removed obsolete sign field; renamed Variable.importT to importT_thms;
Wed, 04 Apr 2007 23:29:37 +0200 rebind HOL.refl as refl (hidden by widen.refl);
wenzelm [Wed, 04 Apr 2007 23:29:37 +0200] rev 22597
rebind HOL.refl as refl (hidden by widen.refl);
Wed, 04 Apr 2007 23:29:33 +0200 rep_thm/cterm/ctyp: removed obsolete sign field;
wenzelm [Wed, 04 Apr 2007 23:29:33 +0200] rev 22596
rep_thm/cterm/ctyp: removed obsolete sign field;
Wed, 04 Apr 2007 20:22:32 +0200 make fresh_guess fail if it does not solve the subgoal
narboux [Wed, 04 Apr 2007 20:22:32 +0200] rev 22595
make fresh_guess fail if it does not solve the subgoal
Wed, 04 Apr 2007 19:56:25 +0200 add a few details in the Fst and Snd cases of unicity proof
narboux [Wed, 04 Apr 2007 19:56:25 +0200] rev 22594
add a few details in the Fst and Snd cases of unicity proof
Wed, 04 Apr 2007 18:05:05 +0200 find_first is just an alias
paulson [Wed, 04 Apr 2007 18:05:05 +0200] rev 22593
find_first is just an alias
Wed, 04 Apr 2007 00:13:13 +0200 added print_mode (generic non-sense);
wenzelm [Wed, 04 Apr 2007 00:13:13 +0200] rev 22592
added print_mode (generic non-sense);
Wed, 04 Apr 2007 00:11:26 +0200 improved exception CTERM;
wenzelm [Wed, 04 Apr 2007 00:11:26 +0200] rev 22591
improved exception CTERM; removed obsolete sign_of/sign_of_thm;
Wed, 04 Apr 2007 00:11:23 +0200 removed unused info channel;
wenzelm [Wed, 04 Apr 2007 00:11:23 +0200] rev 22590
removed unused info channel; renamed Output.has_mode to print_mode_active; cleaned-up Output functions;
Wed, 04 Apr 2007 00:11:22 +0200 added print_mode;
wenzelm [Wed, 04 Apr 2007 00:11:22 +0200] rev 22589
added print_mode;
Wed, 04 Apr 2007 00:11:21 +0200 removed unused info channel;
wenzelm [Wed, 04 Apr 2007 00:11:21 +0200] rev 22588
removed unused info channel;
Wed, 04 Apr 2007 00:11:20 +0200 renamed Output.has_mode to print_mode_active;
wenzelm [Wed, 04 Apr 2007 00:11:20 +0200] rev 22587
renamed Output.has_mode to print_mode_active;
Wed, 04 Apr 2007 00:11:18 +0200 tuned comment;
wenzelm [Wed, 04 Apr 2007 00:11:18 +0200] rev 22586
tuned comment;
Wed, 04 Apr 2007 00:11:17 +0200 cleaned-up Output functions;
wenzelm [Wed, 04 Apr 2007 00:11:17 +0200] rev 22585
cleaned-up Output functions; removed unused info channel; moved print_mode to ROOT.ML (generic non-sense);
Wed, 04 Apr 2007 00:11:16 +0200 improved exception CTERM;
wenzelm [Wed, 04 Apr 2007 00:11:16 +0200] rev 22584
improved exception CTERM; added instantiate_cterm; removed obsolete sign_of_thm;
Wed, 04 Apr 2007 00:11:14 +0200 added scanwords from library.ML (for obsolete rename_tac);
wenzelm [Wed, 04 Apr 2007 00:11:14 +0200] rev 22583
added scanwords from library.ML (for obsolete rename_tac);
Wed, 04 Apr 2007 00:11:13 +0200 removed obsolete scanwords (see obsolete tactic.ML:rename_tac for its only use);
wenzelm [Wed, 04 Apr 2007 00:11:13 +0200] rev 22582
removed obsolete scanwords (see obsolete tactic.ML:rename_tac for its only use);
Wed, 04 Apr 2007 00:11:12 +0200 removed dead code;
wenzelm [Wed, 04 Apr 2007 00:11:12 +0200] rev 22581
removed dead code;
Wed, 04 Apr 2007 00:11:10 +0200 cleaned-up Output functions;
wenzelm [Wed, 04 Apr 2007 00:11:10 +0200] rev 22580
cleaned-up Output functions;
Wed, 04 Apr 2007 00:11:08 +0200 eliminated obsolete rename_tac;
wenzelm [Wed, 04 Apr 2007 00:11:08 +0200] rev 22579
eliminated obsolete rename_tac;
Wed, 04 Apr 2007 00:11:03 +0200 removed obsolete sign_of/sign_of_thm;
wenzelm [Wed, 04 Apr 2007 00:11:03 +0200] rev 22578
removed obsolete sign_of/sign_of_thm;
Wed, 04 Apr 2007 00:10:59 +0200 ML antiquotes;
wenzelm [Wed, 04 Apr 2007 00:10:59 +0200] rev 22577
ML antiquotes;
Tue, 03 Apr 2007 19:31:48 +0200 tuned comments;
wenzelm [Tue, 03 Apr 2007 19:31:48 +0200] rev 22576
tuned comments;
Tue, 03 Apr 2007 19:24:22 +0200 fixed chr/explode;
wenzelm [Tue, 03 Apr 2007 19:24:22 +0200] rev 22575
fixed chr/explode;
Tue, 03 Apr 2007 19:24:21 +0200 avoid overloaded integer constants (accomodate Alice);
wenzelm [Tue, 03 Apr 2007 19:24:21 +0200] rev 22574
avoid overloaded integer constants (accomodate Alice);
Tue, 03 Apr 2007 19:24:19 +0200 avoid clash with Alice keywords;
wenzelm [Tue, 03 Apr 2007 19:24:19 +0200] rev 22573
avoid clash with Alice keywords;
Tue, 03 Apr 2007 19:24:18 +0200 signature: eqtype to accomodate Alice;
wenzelm [Tue, 03 Apr 2007 19:24:18 +0200] rev 22572
signature: eqtype to accomodate Alice;
Tue, 03 Apr 2007 19:24:17 +0200 renamed comp to compose (avoid clash with Alice keywords);
wenzelm [Tue, 03 Apr 2007 19:24:17 +0200] rev 22571
renamed comp to compose (avoid clash with Alice keywords);
Tue, 03 Apr 2007 19:24:16 +0200 renamed of_sort_derivation record fields (avoid clash with Alice keywords);
wenzelm [Tue, 03 Apr 2007 19:24:16 +0200] rev 22570
renamed of_sort_derivation record fields (avoid clash with Alice keywords);
Tue, 03 Apr 2007 19:24:15 +0200 added ML-Systems/alice.ML;
wenzelm [Tue, 03 Apr 2007 19:24:15 +0200] rev 22569
added ML-Systems/alice.ML;
Tue, 03 Apr 2007 19:24:13 +0200 renamed Variable.import to import_thms (avoid clash with Alice keywords);
wenzelm [Tue, 03 Apr 2007 19:24:13 +0200] rev 22568
renamed Variable.import to import_thms (avoid clash with Alice keywords);
Tue, 03 Apr 2007 19:24:11 +0200 removed assert/deny (avoid clash with Alice keywords and confusion due to strict evaluation);
wenzelm [Tue, 03 Apr 2007 19:24:11 +0200] rev 22567
removed assert/deny (avoid clash with Alice keywords and confusion due to strict evaluation);
Tue, 03 Apr 2007 19:24:10 +0200 ranamed CodegenData.lazy to lazy_thms (avoid clash with Alice keywords);
wenzelm [Tue, 03 Apr 2007 19:24:10 +0200] rev 22566
ranamed CodegenData.lazy to lazy_thms (avoid clash with Alice keywords);
Tue, 03 Apr 2007 17:05:52 +0200 remove the lemma swap_fun which was not needed
narboux [Tue, 03 Apr 2007 17:05:52 +0200] rev 22565
remove the lemma swap_fun which was not needed
Tue, 03 Apr 2007 16:20:34 +0200 slighltly improved the proof of unicity
narboux [Tue, 03 Apr 2007 16:20:34 +0200] rev 22564
slighltly improved the proof of unicity
Tue, 03 Apr 2007 12:12:42 +0200 Compatibility file for Alice 1.3 -- experimental!
wenzelm [Tue, 03 Apr 2007 12:12:42 +0200] rev 22563
Compatibility file for Alice 1.3 -- experimental!
Mon, 02 Apr 2007 23:24:52 +0200 rename bij and fresh into bijs and freshs and lookup for eqvts lemma using the ml value instead of the name
narboux [Mon, 02 Apr 2007 23:24:52 +0200] rev 22562
rename bij and fresh into bijs and freshs and lookup for eqvts lemma using the ml value instead of the name
Mon, 02 Apr 2007 11:31:08 +0200 optimizing the null instantiation case
paulson [Mon, 02 Apr 2007 11:31:08 +0200] rev 22561
optimizing the null instantiation case
Mon, 02 Apr 2007 11:30:44 +0200 now exports distinct_subgoal_tac (needed by MetisAPI)
paulson [Mon, 02 Apr 2007 11:30:44 +0200] rev 22560
now exports distinct_subgoal_tac (needed by MetisAPI)
Mon, 02 Apr 2007 11:29:44 +0200 exception handling
paulson [Mon, 02 Apr 2007 11:29:44 +0200] rev 22559
exception handling
Sun, 01 Apr 2007 14:28:48 +0200 added reserved words mod, div for SML
haftmann [Sun, 01 Apr 2007 14:28:48 +0200] rev 22558
added reserved words mod, div for SML
Sat, 31 Mar 2007 15:13:52 +0200 added pt_bij' to the collection perm_swap and also added abs_perm to the collection of equivariance lemmas
urbanc [Sat, 31 Mar 2007 15:13:52 +0200] rev 22557
added pt_bij' to the collection perm_swap and also added abs_perm to the collection of equivariance lemmas
Sat, 31 Mar 2007 12:40:55 +0200 Fixed bug in dest_prem: premises of the form "p x_1 ... x_n"
berghofe [Sat, 31 Mar 2007 12:40:55 +0200] rev 22556
Fixed bug in dest_prem: premises of the form "p x_1 ... x_n" (where p is a variable) are now treated as side conditions if p is not in the list of (global) parameters.
Sat, 31 Mar 2007 08:22:14 +0200 fixed typo
haftmann [Sat, 31 Mar 2007 08:22:14 +0200] rev 22555
fixed typo
Fri, 30 Mar 2007 16:19:03 +0200 simplified constant representation in code generator
haftmann [Fri, 30 Mar 2007 16:19:03 +0200] rev 22554
simplified constant representation in code generator
Fri, 30 Mar 2007 16:19:02 +0200 tuned
haftmann [Fri, 30 Mar 2007 16:19:02 +0200] rev 22553
tuned
Fri, 30 Mar 2007 16:19:01 +0200 equality on strings
haftmann [Fri, 30 Mar 2007 16:19:01 +0200] rev 22552
equality on strings
Fri, 30 Mar 2007 16:19:00 +0200 paraphrasing equality
haftmann [Fri, 30 Mar 2007 16:19:00 +0200] rev 22551
paraphrasing equality
Fri, 30 Mar 2007 16:18:59 +0200 updated
haftmann [Fri, 30 Mar 2007 16:18:59 +0200] rev 22550
updated
Thu, 29 Mar 2007 14:21:47 +0200 improved character output for SML
haftmann [Thu, 29 Mar 2007 14:21:47 +0200] rev 22549
improved character output for SML
Thu, 29 Mar 2007 14:21:45 +0200 dropped legacy ML bindings
haftmann [Thu, 29 Mar 2007 14:21:45 +0200] rev 22548
dropped legacy ML bindings
Thu, 29 Mar 2007 11:59:54 +0200 simplified some steps
paulson [Thu, 29 Mar 2007 11:59:54 +0200] rev 22547
simplified some steps
Thu, 29 Mar 2007 11:12:39 +0200 MESON tactical takes an additional argument: the clausification function.
paulson [Thu, 29 Mar 2007 11:12:39 +0200] rev 22546
MESON tactical takes an additional argument: the clausification function.
Thu, 29 Mar 2007 11:12:03 +0200 Now checks for types-only clause before outputting.
paulson [Thu, 29 Mar 2007 11:12:03 +0200] rev 22545
Now checks for types-only clause before outputting.
Wed, 28 Mar 2007 19:18:39 +0200 - Improved error messages in equivariance proof
berghofe [Wed, 28 Mar 2007 19:18:39 +0200] rev 22544
- Improved error messages in equivariance proof - Renamed <predicate>_eqvt to <predicate>.eqvt
Wed, 28 Mar 2007 19:17:40 +0200 Renamed induct(s)_weak to weak_induct(s) in order to unify
berghofe [Wed, 28 Mar 2007 19:17:40 +0200] rev 22543
Renamed induct(s)_weak to weak_induct(s) in order to unify naming scheme with the one used in nominal_inductive.
Wed, 28 Mar 2007 19:16:11 +0200 - Renamed <predicate>_eqvt to <predicate>.eqvt
berghofe [Wed, 28 Mar 2007 19:16:11 +0200] rev 22542
- Renamed <predicate>_eqvt to <predicate>.eqvt - Renamed induct_weak to weak_induct
Wed, 28 Mar 2007 18:25:23 +0200 the name for the collection of equivariance lemmas is now eqvts (changed from eqvt) in order to avoid clashes with eqvt-lemmas generated in nominal_inductive
urbanc [Wed, 28 Mar 2007 18:25:23 +0200] rev 22541
the name for the collection of equivariance lemmas is now eqvts (changed from eqvt) in order to avoid clashes with eqvt-lemmas generated in nominal_inductive
Wed, 28 Mar 2007 17:27:44 +0200 adapted to new nominal_inductive
urbanc [Wed, 28 Mar 2007 17:27:44 +0200] rev 22540
adapted to new nominal_inductive
Wed, 28 Mar 2007 10:47:19 +0200 Improved code generator for characters: now handles
berghofe [Wed, 28 Mar 2007 10:47:19 +0200] rev 22539
Improved code generator for characters: now handles non-printable characters as well.
Wed, 28 Mar 2007 01:55:18 +0200 tuned proofs (taking full advantage of nominal_inductive)
urbanc [Wed, 28 Mar 2007 01:55:18 +0200] rev 22538
tuned proofs (taking full advantage of nominal_inductive)
Wed, 28 Mar 2007 01:29:43 +0200 adapted to nominal_inductive infrastructure
urbanc [Wed, 28 Mar 2007 01:29:43 +0200] rev 22537
adapted to nominal_inductive infrastructure
Wed, 28 Mar 2007 01:09:23 +0200 made the type sets instance of the "cp" type-class
urbanc [Wed, 28 Mar 2007 01:09:23 +0200] rev 22536
made the type sets instance of the "cp" type-class
Tue, 27 Mar 2007 19:39:40 +0200 added extended the lemma for equivariance of freshness
urbanc [Tue, 27 Mar 2007 19:39:40 +0200] rev 22535
added extended the lemma for equivariance of freshness
Tue, 27 Mar 2007 19:13:28 +0200 adapted to nominal_inductive
urbanc [Tue, 27 Mar 2007 19:13:28 +0200] rev 22534
adapted to nominal_inductive
Tue, 27 Mar 2007 18:28:22 +0200 adapted to new nominal_inductive infrastructure
urbanc [Tue, 27 Mar 2007 18:28:22 +0200] rev 22533
adapted to new nominal_inductive infrastructure
Tue, 27 Mar 2007 17:57:42 +0200 Adapted to new syntax of nominal_inductive.
berghofe [Tue, 27 Mar 2007 17:57:42 +0200] rev 22532
Adapted to new syntax of nominal_inductive.
Tue, 27 Mar 2007 17:57:05 +0200 Adapted to changes in nominal_inductive.
berghofe [Tue, 27 Mar 2007 17:57:05 +0200] rev 22531
Adapted to changes in nominal_inductive.
Tue, 27 Mar 2007 17:55:09 +0200 Implemented proof of strong induction rule.
berghofe [Tue, 27 Mar 2007 17:55:09 +0200] rev 22530
Implemented proof of strong induction rule.
Tue, 27 Mar 2007 17:54:37 +0200 Exported perm_of_pair, mk_not_sym, and perm_simproc.
berghofe [Tue, 27 Mar 2007 17:54:37 +0200] rev 22529
Exported perm_of_pair, mk_not_sym, and perm_simproc.
Tue, 27 Mar 2007 12:28:42 +0200 cleaned up HOL/ex/Code*.thy
haftmann [Tue, 27 Mar 2007 12:28:42 +0200] rev 22528
cleaned up HOL/ex/Code*.thy
Tue, 27 Mar 2007 09:19:37 +0200 fixed document preparation
haftmann [Tue, 27 Mar 2007 09:19:37 +0200] rev 22527
fixed document preparation
Mon, 26 Mar 2007 16:35:33 +0200 fixed problem with mutual recursion
krauss [Mon, 26 Mar 2007 16:35:33 +0200] rev 22526
fixed problem with mutual recursion
Mon, 26 Mar 2007 14:54:45 +0200 cleaned up Library/ and ex/
haftmann [Mon, 26 Mar 2007 14:54:45 +0200] rev 22525
cleaned up Library/ and ex/
Mon, 26 Mar 2007 14:53:07 +0200 minimal intro rules
haftmann [Mon, 26 Mar 2007 14:53:07 +0200] rev 22524
minimal intro rules
Mon, 26 Mar 2007 14:53:06 +0200 exported interface for intro rules
haftmann [Mon, 26 Mar 2007 14:53:06 +0200] rev 22523
exported interface for intro rules
(0) -10000 -3000 -1000 -300 -100 -96 +96 +100 +300 +1000 +3000 +10000 +30000 tip