Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-3000
-1000
-128
+128
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
adapted to new PureThy.add_defs;
1998-04-29, by wenzelm
Theory.require;
1998-04-29, by wenzelm
tuned setup;
1998-04-29, by wenzelm
tuned setup;
1998-04-29, by wenzelm
tuned names of (add_)store_XXX functions;
1998-04-29, by wenzelm
replaced thy_setup by 'setup' section;
1998-04-29, by wenzelm
added append;
1998-04-29, by wenzelm
added none: 'a -> 'a * 'b attribute list;
1998-04-29, by wenzelm
tuned error msgs;
1998-04-29, by wenzelm
moved mk_defpair to logic.ML;
1998-04-29, by wenzelm
tuned get_ax (uses ancestry);
1998-04-29, by wenzelm
renamed setup to apply;
1998-04-29, by wenzelm
adapted to new PureThy.add_axioms_i;
1998-04-29, by wenzelm
added defaultS: sg -> sort;
1998-04-29, by wenzelm
added thm, thms;
1998-04-29, by wenzelm
*** empty log message ***
1998-04-29, by wenzelm
new thms, really demos of the final coalgebra theorem
1998-04-28, by paulson
new thms image_0_left, image_Un_left, etc.
1998-04-28, by paulson
new thm mult_lt_mono1
1998-04-28, by paulson
cleanup for split_all_tac as wrapper in claset()
1998-04-27, by oheimb
removed wrong comment
1998-04-27, by oheimb
added option_map_eq_Some via AddIffs
1998-04-27, by oheimb
*** empty log message ***
1998-04-27, by nipkow
delsplits, Addsplits, Delsplits.
1998-04-27, by nipkow
Renamed expand_const -> split_const
1998-04-27, by nipkow
Added conversion of reg.expr. to automata.
1998-04-27, by nipkow
Renamed expand_const -> split_const.
1998-04-27, by nipkow
Added a few lemmas.
1998-04-27, by nipkow
New proof of apply_equality and new thm Pi_image_cons
1998-04-27, by paulson
improved split_all_tac significantly
1998-04-24, by oheimb
improved keyboard modifiers
1998-04-24, by oheimb
added ASCII translation of subseteq
1998-04-24, by oheimb
tidied; div & mod
1998-04-24, by paulson
*** empty log message ***
1998-04-24, by oheimb
added no_syn;
1998-04-22, by wenzelm
added mk_cond_defpair, mk_defpair;
1998-04-22, by wenzelm
Modifications due to improved simplifier.
1998-04-22, by nipkow
Tried to speed up the rewriter by eta-contracting all patterns beforehand and
1998-04-22, by nipkow
improved pair_tac to call prune_params_tac afterwards
1998-04-21, by oheimb
split_all_tac is now added to claset() _before_ other safe tactics
1998-04-21, by oheimb
made proof of zmult_congruent2 more stable
1998-04-21, by oheimb
simplification of explicit theory usage and merges
1998-04-21, by oheimb
removed split_all_tac from claset() globally within IOA
1998-04-21, by oheimb
made modifications of the simpset() local
1998-04-21, by oheimb
layout improvement
1998-04-21, by oheimb
expandshort; new gcd_induct with inbuilt case analysis
1998-04-21, by paulson
Renamed mod_XXX_cancel to mod_XXX_self
1998-04-21, by paulson
New laws for mod
1998-04-20, by paulson
proving fib(gcd(m,n)) = gcd(fib m, fib n)
1998-04-20, by paulson
fixed comment;
1998-04-19, by wenzelm
Fixed bug in inductive sections to allow disjunctive premises;
1998-04-10, by paulson
bug fixes
1998-04-10, by paulson
can prove the empty relation to be WF
1998-04-10, by paulson
Fixed bug in inductive sections to allow disjunctive premises;
1998-04-10, by paulson
Clearer description of recdef, including use of {}
1998-04-09, by paulson
Simplified the syntax description; mentioned FOL vs HOL
1998-04-09, by paulson
*** empty log message ***
1998-04-07, by oheimb
replaced option_map_SomeD by option_map_eq_Some (RS iffD1)
1998-04-07, by oheimb
made split_all_tac as safe wrapper more defensive:
1998-04-07, by oheimb
no open Simplifier;
1998-04-04, by wenzelm
tuned fail;
1998-04-04, by wenzelm
type_error;
1998-04-04, by wenzelm
tuned comments;
1998-04-04, by wenzelm
no open Simplifier;
1998-04-04, by wenzelm
replaced thy_data by thy_setup;
1998-04-04, by wenzelm
type_error;
1998-04-04, by wenzelm
replaced thy_data by setup;
1998-04-04, by wenzelm
removed simple;
1998-04-04, by wenzelm
added triv_goal, rev_triv_goal (for Isar);
1998-04-04, by wenzelm
added Goal_def;
1998-04-04, by wenzelm
replaced thy_data by thy_setup;
1998-04-04, by wenzelm
added local_theory (for Isar);
1998-04-04, by wenzelm
tuned trace msgs;
1998-04-04, by wenzelm
tuned names;
1998-04-03, by wenzelm
added get_tthm(s), store_tthms(s);
1998-04-03, by wenzelm
tuned comments;
1998-04-03, by wenzelm
added attribute.ML;
1998-04-03, by wenzelm
Theorem tags and attributes.
1998-04-03, by wenzelm
UNITY
1998-04-03, by paulson
repaired incompatibility with new SML version by eta-expansion
1998-04-03, by oheimb
New target HOL-UNITY
1998-04-03, by paulson
New UNITY theory
1998-04-03, by paulson
Tidied proofs
1998-04-03, by paulson
Tidied proofs by getting rid of case_tac
1998-04-03, by paulson
improved \tt appearance of many ASCII special symbols like #
1998-04-03, by oheimb
split_all_tac now fails if there is nothing to split
1998-04-02, by oheimb
new theorems
1998-04-02, by paulson
changed if_bool_eq to if_bool_eq_conj
1998-04-02, by paulson
changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
1998-04-02, by paulson
New theorems card_Diff_le and card_insert_le; tidied
1998-04-02, by paulson
introduced functions for updating the wrapper lists
1998-04-02, by oheimb
*** empty log message ***
1998-04-02, by oheimb
merge_cs now also merges safe and unsafe wrappers
1998-03-30, by oheimb
generalized appearance of trancl_into_rtrancl and r_into_trancl
1998-03-30, by oheimb
adapted proof of finite_converse
1998-03-30, by oheimb
added wf_converse_trancl, adapted proof of wfrec
1998-03-30, by oheimb
added caveat
1998-03-30, by oheimb
added introduction and elimination rules for Univalent
1998-03-30, by oheimb
added Univalent_rel_pow
1998-03-30, by oheimb
removed superfluous use_thy
1998-03-30, by oheimb
removed superfluous translations
1998-03-30, by oheimb
added try, single, many;
1998-03-24, by wenzelm
added cproj', and therefore extended prj
1998-03-24, by oheimb
added cproj', and therefore extended prj
1998-03-24, by oheimb
improved checks
1998-03-24, by oheimb
added o2s
1998-03-24, by oheimb
added finite_acyclic_wf_converse: corrected 8bit chars
1998-03-24, by oheimb
added acyclicI
1998-03-24, by oheimb
added finite_acyclic_wf_converse
1998-03-24, by oheimb
more thms
1998-03-23, by paulson
inverse -> converse
1998-03-16, by paulson
inverse -> converse
1998-03-16, by paulson
re-ordered proofs
1998-03-16, by paulson
moved addsplits [expand_if] from HOL_basic_ss to HOL_ss;
1998-03-13, by wenzelm
renamed not1_or to disj_not1, not2_or to disj_not2
1998-03-12, by oheimb
improved coding of delWrapper and delSWrapper
1998-03-12, by oheimb
addloop: added warning in case of overwriting a looper
1998-03-12, by oheimb
Made mutual simplification of prems a special case.
1998-03-12, by nipkow
Used merge_alists for loopers.
1998-03-12, by nipkow
New, stronger rewrites
1998-03-12, by paulson
The theorem nat_neqE, and some tidying
1998-03-12, by paulson
New laws, mostly generalizing old "pred" ones
1998-03-12, by paulson
spy_analz_tac now handles individual conjuncts properly
1998-03-11, by paulson
new theorem
1998-03-11, by paulson
New theorem Image_eq_UN; deleted the silly vimage_inverse_Image
1998-03-11, by paulson
Arith.thy -> thy; proved a few new theorems
1998-03-11, by paulson
New Asm_full_simp_tac shortens proof.
1998-03-11, by nipkow
Simplifier
1998-03-11, by nipkow
less
more
|
(0)
-3000
-1000
-128
+128
+1000
+3000
+10000
+30000
tip