Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-256
+256
+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.
tuned;
2012-02-26, by wenzelm
tuned signature;
2012-02-26, by wenzelm
merged
2012-02-25, by wenzelm
slightly changing the enumeration scheme
2012-02-25, by bulwahn
adding some more test invocations of find_unused_assms
2012-02-25, by bulwahn
adding an example where random beats exhaustive testing
2012-02-25, by bulwahn
removing unnecessary assumptions in RComplete;
2012-02-25, by bulwahn
removing unnecessary assumptions in RealDef;
2012-02-25, by bulwahn
one general list_all2_update_cong instead of two special ones
2012-02-25, by bulwahn
tuned comments;
2012-02-25, by wenzelm
standard Graph instances;
2012-02-25, by wenzelm
clarified signature -- avoid oddities of Iterable like Iterator.map;
2012-02-25, by wenzelm
discontinued slightly odd Graph.del_nodes (inefficient due to full Table.map);
2012-02-25, by wenzelm
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
2012-02-24, by haftmann
explicit is better than implicit
2012-02-24, by haftmann
dropped dead code
2012-02-24, by haftmann
prefer sorted Map/Set for canonical order of results -- pass ordering via fresh copy of empty;
2012-02-24, by wenzelm
tuned imports;
2012-02-24, by wenzelm
tuned signature;
2012-02-24, by wenzelm
discontinued obsolete Graph.all_paths (last seen in 1524d69783d3 and AFP/80bbbdbfec62);
2012-02-24, by wenzelm
merged
2012-02-24, by wenzelm
remove ill-formed lemmas word_0_wi_Pls and word_m1_wi_Min
2012-02-24, by huffman
avoid using Int.succ_def in proofs
2012-02-24, by huffman
avoid using Int.succ or Int.pred in proofs
2012-02-24, by huffman
avoid using BIT_simps in proofs;
2012-02-24, by huffman
avoid using BIT_simps in proofs
2012-02-24, by huffman
updated stats according to src/HOL/IsaMakefile;
2012-02-24, by wenzelm
more precise clean target;
2012-02-24, by wenzelm
clarifed name space "type name", which covers logical and non-logical types, and often occurs inside outer syntax "type" markup;
2012-02-24, by wenzelm
avoid using Int.Pls_def in proofs
2012-02-24, by huffman
remove ill-formed lemmas word_pred_0_Min and word_m1_Min
2012-02-24, by huffman
remove ill-formed lemma of_bl_no; adapt proofs
2012-02-24, by huffman
adapt lemma mask_lem to respect int/bin distinction
2012-02-24, by huffman
rephrase some slow "metis" calls
2012-02-24, by blanchet
added support for Alt-Ergo through Why3 (mostly for experimental purposes, e.g. polymorphism vs. monomorphization)
2012-02-24, by blanchet
general solution to the arity bug that occasionally plagues Sledgehammer -- short story, lots of things go kaputt when a polymorphic symbol's arity in the translation is higher than the arity of the fully polymorphic HOL constant
2012-02-24, by blanchet
renamed 'try_methods' to 'try0'
2012-02-24, by blanchet
doc fixes (thanks to Nik)
2012-02-24, by blanchet
fixed arity bug with "If" helpers for "If" that returns a function
2012-02-24, by blanchet
given up disfruitful branch
2012-02-24, by haftmann
explicit remove of lattice notation
2012-02-24, by haftmann
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
2012-02-24, by haftmann
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
2012-02-23, by haftmann
dropped dead code
2012-02-23, by haftmann
tuned isatest settings;
2012-02-23, by wenzelm
merged
2012-02-23, by wenzelm
moved lemmas for orderings and lattices on predicates to corresponding theories, retaining declaration order of classical rules; tuned headings; tuned syntax
2012-02-23, by haftmann
tuned whitespace
2012-02-23, by haftmann
tuned proof
2012-02-23, by haftmann
prefer actual syntax categories;
2012-02-23, by wenzelm
avoid trait Addable, which is deprecated in scala-2.9.x;
2012-02-23, by wenzelm
streamlined abstract datatype;
2012-02-23, by wenzelm
tuned;
2012-02-23, by wenzelm
streamlined abstract datatype;
2012-02-23, by wenzelm
tuned -- avoid copy of empty value;
2012-02-23, by wenzelm
tuned;
2012-02-23, by wenzelm
streamlined abstract datatype, eliminating odd representation class;
2012-02-23, by wenzelm
tuned;
2012-02-23, by wenzelm
merged
2012-02-23, by huffman
make more simp rules respect int/bin distinction
2012-02-23, by huffman
make bool list functions respect int/bin distinction
2012-02-23, by huffman
merged;
2012-02-23, by wenzelm
tuned;
2012-02-23, by wenzelm
clarified Graph.restrict (formerly Graph.subgraph) based on public graph operations;
2012-02-23, by wenzelm
further graph operations from ML;
2012-02-23, by wenzelm
removed dead code;
2012-02-23, by wenzelm
directed graphs (in Scala);
2012-02-23, by wenzelm
make uses of bin_split respect int/bin distinction
2012-02-23, by huffman
remove lemma bin_cat_Pls, which doesn't respect int/bin distinction
2012-02-23, by huffman
make uses of constant bin_sc respect int/bin distinction
2012-02-23, by huffman
remove duplicate lemma bintrunc_Suc in favor of bintrunc.Suc
2012-02-23, by huffman
remove unused lemmas
2012-02-23, by huffman
simplify proofs
2012-02-23, by huffman
make uses of bin_sign respect int/bin distinction
2012-02-23, by huffman
removed unnecessary lemma zero_bintrunc
2012-02-23, by huffman
remove unnecessary lemmas
2012-02-23, by huffman
removed unnecessary constant bin_rl
2012-02-23, by huffman
remove duplication of lemmas bin_{rest,last}_BIT
2012-02-23, by huffman
remove lemmas Bit{0,1}_div2
2012-02-23, by huffman
simplify proof
2012-02-23, by huffman
deal with FIXMEs for linarith examples
2012-02-23, by huffman
CONTRIBUTORS
2012-02-23, by haftmann
merged
2012-02-22, by huffman
tuned whitespace
2012-02-22, by huffman
tuned whitespace
2012-02-22, by huffman
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
2012-02-22, by bulwahn
NEWS
2012-02-22, by bulwahn
adding some examples with find_unused_assms command
2012-02-22, by bulwahn
adding new command "find_unused_assms"
2012-02-22, by bulwahn
removing some unnecessary premises from Map theory
2012-02-22, by bulwahn
preliminarily switching quickcheck-narrowing off by default (probably it should only be invoked if concrete testing does not work)
2012-02-22, by bulwahn
generalizing inj_on_Int
2012-02-22, by bulwahn
moving Quickcheck's example to its own session
2012-02-22, by bulwahn
tuned proofs;
2012-02-21, by wenzelm
more robust visible_range: allow empty view;
2012-02-21, by wenzelm
misc tuning;
2012-02-21, by wenzelm
merged;
2012-02-21, by wenzelm
made SML/NJ happy;
2012-02-21, by wenzelm
tuned proofs;
2012-02-21, by wenzelm
merged
2012-02-21, by wenzelm
tuned proofs;
2012-02-21, by wenzelm
approximate Perspective.full within the bounds of the JVM;
2012-02-21, by wenzelm
misc tuning;
2012-02-21, by wenzelm
invoke later to reduce chance of causing deadlock;
2012-02-21, by wenzelm
misc tuning;
2012-02-21, by wenzelm
separate module for text status overview;
2012-02-21, by wenzelm
overview.delay_repaint: avoid wasting GUI cycles via update_delay;
2012-02-21, by wenzelm
tuned;
2012-02-21, by wenzelm
merged
2012-02-21, by berghofe
merged
2012-02-21, by berghofe
Fixed bugs:
2012-02-20, by berghofe
merged
2012-02-21, by bulwahn
subtype preprocessing in Quickcheck;
2012-02-21, by bulwahn
adding parsing of an optional predicate with quickcheck_generator command
2012-02-21, by bulwahn
updated generated files (cf. 8d51b375e926);
2012-02-21, by wenzelm
merged;
2012-02-21, by wenzelm
add missing lemmas to compute_div_mod
2012-02-21, by huffman
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
2012-02-21, by huffman
avoid using constant Int.neg
2012-02-21, by huffman
renamed ex/Numeral.thy to ex/Numeral_Representation.thy
2012-02-21, by huffman
reverting changesets from 5d33a3269029 on: change of order of declaration of classical rules makes serious problems
2012-02-21, by haftmann
tuned whitespace
2012-02-20, by haftmann
tuned proof
2012-02-20, by haftmann
tuned proof
2012-02-19, by haftmann
distributed lattice properties of predicates to places of instantiation
2012-02-19, by haftmann
removing some unnecessary premises from Divides
2012-02-20, by bulwahn
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
2012-02-20, by huffman
observe HEIGHT of overview ticks;
2012-02-20, by wenzelm
more careful painting of overview component: more precise and more efficient;
2012-02-20, by wenzelm
clarified initial process startup errors: recover image load failure message (cf. 2cb7e34f6096) and suppress accidental output from raw ML toplevel;
2012-02-20, by wenzelm
use qualified constant names instead of suffixes (from Florian Haftmann)
2012-02-20, by huffman
tuned proofs
2012-02-18, by haftmann
tuned
2012-02-12, by haftmann
brute-force adjustion
2012-02-11, by haftmann
tuned whitespace
2012-02-11, by haftmann
tuned
2012-02-11, by haftmann
tuned
2012-02-10, by haftmann
tuned code
2012-02-10, by haftmann
dropped whitespace
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
corrected typo
2012-02-10, by haftmann
dropped dead code
2012-02-10, by haftmann
notepad is more appropriate here
2012-02-12, by haftmann
corrected treatment of applications of built-in functions to higher-order terms
2012-02-18, by boehmes
NEWS
2012-02-18, by krauss
merged
2012-02-18, by krauss
added congruence rules for Option.{map|bind}
2012-02-18, by krauss
updated generated documents
2012-02-18, by haftmann
avoid redefinition of @{theory} antiquotation
2012-02-18, by haftmann
update of generated documents
2012-02-18, by haftmann
tuned whitespace
2012-02-18, by haftmann
clarified
2012-02-18, by haftmann
corrected spelling
2012-02-18, by haftmann
clarified
2012-02-18, by haftmann
more precise semantics of "theory" antiquotation
2012-02-18, by haftmann
tuned import
2012-02-18, by haftmann
dropped references to obsolete theories
2012-02-18, by haftmann
adjusted to set type constructor
2012-02-18, by haftmann
tuned whitespace
2012-02-18, by haftmann
more explicit error on malformed abstract equation; dropped dead code; tuned signature
2012-02-18, by haftmann
simplified configuration options for syntax ambiguity;
2012-02-17, by wenzelm
retain default of Syntax.ambiguity, according to 2bd54d4b5f3d (despite earlier versions);
2012-02-17, by wenzelm
more antiquotations;
2012-02-16, by wenzelm
more symbols;
2012-02-16, by wenzelm
tuned imports;
2012-02-16, by wenzelm
tuned proofs;
2012-02-16, by wenzelm
simplified configuration options for syntax ambiguity;
2012-02-16, by wenzelm
merged
2012-02-16, by wenzelm
removing unnecessary premise from diff_single_insert
2012-02-16, by bulwahn
explicit is better than implicit;
2012-02-16, by wenzelm
more uniform / portable representation of the idea of "copy_dir" (NB: cp -f dereferences symlinks on GNU/Linux, but does not on old-school Unixen including BSD/Mac OS X);
2012-02-16, by wenzelm
simplifying proof
2012-02-16, by bulwahn
removing unnecessary premises in theorems of List theory
2012-02-16, by bulwahn
tuning mutabelle script
2012-02-16, by bulwahn
adding documentation for abort_potential option in quickcheck
2012-02-16, by bulwahn
renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
2012-02-15, by wenzelm
discontinued Drule.term_rule, which tends to cause confusion due to builtin cterm_of (NB: the standard morphisms already provide a separate term component);
2012-02-15, by wenzelm
uniform Isar source formatting for this file;
2012-02-15, by wenzelm
clarified outer syntax "constdecl", which is only local to some rail diagrams;
2012-02-15, by wenzelm
discontinued obsolete "prems" fact;
2012-02-15, by wenzelm
eliminated slightly odd / obsolete DETERM_UNTIL, DETERM_UNTIL_SOLVED (cf. 941afb897532, ea0668a1c0ba);
2012-02-15, by wenzelm
removed obsolete files;
2012-02-15, by wenzelm
more basic simplification, eliminated slightly odd tactic style from 1995 (cf. ea0668a1c0ba);
2012-02-15, by wenzelm
removed dead code;
2012-02-15, by wenzelm
updated listrel (cf. 80dccedd6c14);
2012-02-15, by wenzelm
removed redundant cut_inst_tac -- already covered in implementation manual;
2012-02-15, by wenzelm
updated rewrite_goals_rule, rewrite_rule;
2012-02-15, by wenzelm
NEWS;
2012-02-15, by wenzelm
updated refs;
2012-02-15, by wenzelm
renamed "xstr" to "str_token";
2012-02-15, by wenzelm
merged
2012-02-14, by wenzelm
don't report spurious LEO-II errors
2012-02-14, by blanchet
better error message
2012-02-14, by blanchet
removing debug code in mutabelle
2012-02-14, by bulwahn
adding abort_potential functionality in quickcheck
2012-02-14, by bulwahn
adding abort_potential configuration in Quickcheck
2012-02-14, by bulwahn
clarified bires_inst_tac: retain internal exceptions;
2012-02-14, by wenzelm
tuned signature;
2012-02-14, by wenzelm
more conventional tactic setup -- avoid low-level Thm.dest_state and spurious warnings about it;
2012-02-14, by wenzelm
more conventional tactic setup;
2012-02-14, by wenzelm
eliminated odd/obsolete innermost_params (cf. a77ad6c86564, 3458b0e955ac);
2012-02-14, by wenzelm
prefer high-level elim_format;
2012-02-14, by wenzelm
discontinued unused MRL -- in correspondence with section "2.4.2 Rule composition" in the implementation manual;
2012-02-14, by wenzelm
method setup;
2012-02-14, by wenzelm
simplified use of tacticals;
2012-02-14, by wenzelm
comment;
2012-02-14, by wenzelm
tuned signature, according to actual usage of these operations;
2012-02-14, by wenzelm
tuned signature;
2012-02-14, by wenzelm
normalized aliases;
2012-02-14, by wenzelm
elininated unused INTLEAVE;
2012-02-14, by wenzelm
eliminated unused rewrite_goal_rule;
2012-02-14, by wenzelm
eliminated unused subgoals_tac;
2012-02-14, by wenzelm
eliminated obsolete aliases;
2012-02-14, by wenzelm
eliminated obsolete aliases;
2012-02-14, by wenzelm
tuned;
2012-02-14, by wenzelm
merged, resolving trivial conflicts;
2012-02-14, by wenzelm
merged;
2012-02-14, by wenzelm
new SPASS options
2012-02-11, by blanchet
making num_mutations a configuration that can be changed with the mutabelle bash command
2012-02-11, by bulwahn
making max_mutants an option that can be changed in the Mutabelle-script
2012-02-11, by bulwahn
increase timeout to 30 seconds; changing mutabelle script
2012-02-11, by bulwahn
parse clauses generated from several formulas
2012-02-10, by blanchet
be more gentle when generating KBO weights
2012-02-10, by blanchet
update SPASS slices
2012-02-10, by blanchet
more specification of the quotient package in IsarRef
2012-02-10, by Cezary Kaliszyk
specification of the quotient package
2012-02-10, by Cezary Kaliszyk
tune KBO weight code
2012-02-09, by blanchet
minor DFG fix
2012-02-09, by blanchet
new SPASS slices
2012-02-09, by blanchet
improved KBO weights -- beware of explicit applications
2012-02-09, by blanchet
added possibility of generating KBO weights to DFG problems
2012-02-09, by blanchet
Generalize the compositional preservation theorems
2012-02-09, by Cezary Kaliszyk
use 'primrec' to define "rotate1", for uniformity (and to help first-order tools that rely on "Spec_Rules")
2012-02-08, by blanchet
removed fact that confuses SPASS -- better rely on "rev_rev_ident", which is stronger and more ATP friendly
2012-02-08, by blanchet
beware of "Bit0" and "Bit1" -- these shouldn't be blidly unfolded by SPASS, lest we get gigantic terms
2012-02-08, by blanchet
fixed arity error
2012-02-06, by blanchet
tuning
2012-02-06, by blanchet
renamed type encoding
2012-02-06, by blanchet
adding some forbidden constant names for mutabelle
2012-02-05, by bulwahn
mutabelle ignores theorems with internal constants
2012-02-05, by bulwahn
tuned
2012-02-05, by nipkow
merged
2012-02-05, by nipkow
simplified code generation
2012-02-05, by nipkow
remove option that's on by default
2012-02-05, by blanchet
no need for a script/mega-hack with the new SPASS
2012-02-05, by blanchet
cleaned up new SPASS parsing
2012-02-05, by blanchet
tuning
2012-02-05, by blanchet
merged
2012-02-05, by bulwahn
adding code equation for Relation.image; adding map_project as correspondence to map_filter on lists
2012-02-05, by bulwahn
tuning to remove ML warnings
2012-02-05, by bulwahn
removed double filtering of type args
2012-02-05, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-256
+256
+1000
+3000
+10000
+30000
tip