Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-112
+112
+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.
TypeExt.decode_term;
2007-04-21, by wenzelm
added decode_term (belongs to Syntax module);
2007-04-21, by wenzelm
tuned the setup of fresh_fun
2007-04-21, by urbanc
defs are added to code data
2007-04-20, by haftmann
repaired value restriction problem
2007-04-20, by haftmann
reverted to classical syntax for K_record
2007-04-20, by haftmann
tuned
2007-04-20, by haftmann
Interpretation equations applied to attributes
2007-04-20, by ballarin
Interpretation equations applied to attributes;
2007-04-20, by ballarin
Modified eqvt_tac to avoid failure due to introduction rules
2007-04-20, by berghofe
clarifed
2007-04-20, by haftmann
modify fresh_fun_simp to ease debugging
2007-04-20, by narboux
updated code generator
2007-04-20, by haftmann
updated
2007-04-20, by haftmann
adds extracted program to code theorem table
2007-04-20, by haftmann
unfold attribute now also accepts HOL equations
2007-04-20, by haftmann
added more stuff
2007-04-20, by haftmann
add definitions explicitly to code generator table
2007-04-20, by haftmann
cleared dead code
2007-04-20, by haftmann
moved axclass module closer to core system
2007-04-20, by haftmann
Isar definitions are now added explicitly to code theorem table
2007-04-20, by haftmann
improved case unfolding
2007-04-20, by haftmann
switched from recdef to function package; constants add, mul, pow now curried; infix syntax for algebraic operations.
2007-04-20, by haftmann
tuned syntax: K_record is now an authentic constant
2007-04-20, by haftmann
tuned: now using function package
2007-04-20, by haftmann
transfer_tac accepts also HOL equations as theorems
2007-04-20, by haftmann
shifted min/max to class order
2007-04-20, by haftmann
tuned
2007-04-20, by haftmann
added class tutorial
2007-04-20, by haftmann
code generator changes
2007-04-20, by haftmann
generate page labels
2007-04-20, by krauss
definition lookup via terms, not names. Methods "relation" and "lexicographic_order"
2007-04-20, by krauss
declared lemmas true_eqvt and false_eqvt to be equivariant (suggested by samth at ccs.neu.edu)
2007-04-20, by urbanc
trying to make single-step proofs work better, especially if they contain
2007-04-19, by paulson
nominal_inductive no longer proves equivariance.
2007-04-19, by berghofe
add a tactic to generate fresh names
2007-04-19, by narboux
simplified ProofContext.infer_types(_pats);
2007-04-18, by wenzelm
Improved comments.
2007-04-18, by dixon
proper header, added regression tests
2007-04-18, by krauss
added temporary hack to avoid schematic goals in "termination".
2007-04-18, by krauss
Fixes for proof reconstruction, especially involving abstractions and definitions
2007-04-18, by paulson
export is_dummy_pattern;
2007-04-17, by wenzelm
lemma isCont_inv_fun is same as isCont_inverse_function
2007-04-17, by huffman
moved root and sqrt lemmas from Transcendental.thy to NthRoot.thy
2007-04-17, by huffman
remove use of pos_boundedE
2007-04-17, by huffman
lemma geometric_sum no longer needs class division_by_zero
2007-04-17, by huffman
tuned proofs;
2007-04-17, by wenzelm
canonical merge operations
2007-04-16, by haftmann
added print_indexname;
2007-04-16, by wenzelm
improved the equivariance lemmas for the quantifiers; had to export the lemma eqvt_force_add and eqvt_force_del in the thmdecls
2007-04-16, by urbanc
added a more usuable lemma for dealing with fresh_fun
2007-04-16, by urbanc
generalized type of lemma geometric_sum
2007-04-16, by huffman
replaced read_term_legacy by read_prop_legacy;
2007-04-15, by wenzelm
removed obsolete redeclare_skolems;
2007-04-15, by wenzelm
read prop as prop, not term;
2007-04-15, by wenzelm
removed obsolete TypeInfer.logicT -- use dummyT;
2007-04-15, by wenzelm
avoid internal names;
2007-04-15, by wenzelm
tuned;
2007-04-15, by wenzelm
legacy_infer_term/prop -- including intern_term;
2007-04-15, by wenzelm
Thm.plain_prop_of;
2007-04-15, by wenzelm
added decode_types (from type_infer.ML);
2007-04-15, by wenzelm
added read_term;
2007-04-15, by wenzelm
added mixfixT (from type_infer.ML);
2007-04-15, by wenzelm
proper interface infer_types(_pat);
2007-04-15, by wenzelm
Thm.fold_terms;
2007-04-15, by wenzelm
removed unused Output.panic hook -- internal to PG wrapper;
2007-04-15, by wenzelm
moved get_sort to sign.ML;
2007-04-15, by wenzelm
removed obsolete inferT_axm;
2007-04-15, by wenzelm
removed obsolete infer_types(_simult);
2007-04-15, by wenzelm
moved Drule.plain_prop_of, Drule.fold_terms to more_thm.ML;
2007-04-15, by wenzelm
load type_infer.ML early;
2007-04-15, by wenzelm
adapted decode_type;
2007-04-15, by wenzelm
proper ProofContext.infer_types;
2007-04-15, by wenzelm
Thm.fold_terms;
2007-04-15, by wenzelm
replaced axioms/finalconsts by proper axiomatization;
2007-04-15, by wenzelm
simplified read_axm;
2007-04-14, by wenzelm
tuned comment;
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
removed redundant string_of_vname (see term.ML);
2007-04-14, by wenzelm
removed obsolete read_ctyp, read_def_cterm;
2007-04-14, by wenzelm
tuned signature;
2007-04-14, by wenzelm
read_typ_XXX: no sorts;
2007-04-14, by wenzelm
added read_def_cterms, read_cterm (from thm.ML);
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
removed Pure/Syntax/ROOT.ML;
2007-04-14, by wenzelm
Term.string_of_vname;
2007-04-14, by wenzelm
Theory.inferT_axm;
2007-04-14, by wenzelm
do not enable Toplevel.debug globally;
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
canonical merge operations
2007-04-14, by haftmann
declarations: apply target_morphism;
2007-04-14, by wenzelm
inst(T)_morphism: avoid reference to static theory value;
2007-04-14, by wenzelm
tuned signature;
2007-04-14, by wenzelm
added Morphism.transform/form (generic non-sense);
2007-04-14, by wenzelm
Morphism.transform/form;
2007-04-14, by wenzelm
data declaration: removed obsolete target_morphism (still required for local data!?);
2007-04-14, by wenzelm
data declaration: removed obsolete target_morphism;
2007-04-14, by wenzelm
added eval_antiquotes_fn (tmp);
2007-04-13, by wenzelm
tuned document (headers, sections, spacing);
2007-04-13, by wenzelm
do translation: CONST;
2007-04-13, by wenzelm
eval_antiquotes: proper parentheses for projection;
2007-04-13, by wenzelm
canonical merge operations
2007-04-13, by haftmann
Removed erroneous application of rev in get_clauses that caused
2007-04-13, by berghofe
more robust proof
2007-04-13, by krauss
Experimental code for the interpretation of definitions.
2007-04-13, by ballarin
Experimental interpretation code for definitions.
2007-04-13, by ballarin
New file for locale regression tests.
2007-04-13, by ballarin
debug versions of finite_guess and fresh_guess do not fail if they can not solve the goal
2007-04-13, by narboux
minimize imports
2007-04-13, by huffman
new simp rule exp_ln; new standard proof of DERIV_exp_ln_one; changed imports
2007-04-13, by huffman
moved nonstandard derivative stuff from Deriv.thy into new file HDeriv.thy
2007-04-13, by huffman
less
more
|
(0)
-10000
-3000
-1000
-112
+112
+1000
+3000
+10000
+30000
tip