Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-512
+512
+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
adding a quickcheck example about functions and sets
2012-02-05, by bulwahn
removing lemma bij_betw_Disj_Un, as it is a special case of bij_between_combine (was added in d1fc454d6735, and has not been used since)
2012-02-05, by bulwahn
adding a remark about lemma which is too special and should be removed
2012-02-05, by bulwahn
another try to improve code generation of set equality (cf. da32cf32c0c7)
2012-02-05, by bulwahn
beautifying definitions of check_all and adding instance for finite_4
2012-02-05, by bulwahn
Make automatic derivation of raw/quotient types more greedy to allow descending and quot_lifted for compound quotients.
2012-02-05, by Cezary Kaliszyk
added option to Mirabelle/Sledgehammer
2012-02-04, by blanchet
improved hashing w.r.t. Mirabelle, to help debugging
2012-02-04, by blanchet
tuned SPASS DFG output
2012-02-04, by blanchet
the new SPASS gives accurate fact information, so no need for old hack anymore
2012-02-04, by blanchet
fixed docs
2012-02-04, by blanchet
made sure to filter type args also for "uncurried alias" equations
2012-02-04, by blanchet
made option available to users (mostly for experiments)
2012-02-04, by blanchet
using fully qualified module names in Haskell source, which seems to be required by GHC 7.0.4 (also cf. 0fd9ab902b5a)
2012-02-04, by bulwahn
optimization: slice caching in case two consecutive slices are nearly identical
2012-02-03, by blanchet
extended SPASS/DFG output with ranks
2012-02-03, by blanchet
try to pass fewer options to Metis
2012-02-03, by blanchet
Quotient FSet: Add compositional respectfulness and preservation for map and lift map_concat
2012-02-03, by Cezary Kaliszyk
improve SPASS scripts
2012-02-02, by blanchet
change 9ce354a77908 wasn't quite right -- here's an improvement
2012-02-02, by blanchet
better SPASS setup
2012-02-02, by blanchet
don't introduce new symbols in helpers -- makes problems unprovable
2012-02-02, by blanchet
only constants can be aliased
2012-02-02, by blanchet
include new SPASS by default if available
2012-02-02, by blanchet
adding an example for finite and cofinite sets
2012-02-02, by bulwahn
adding a minimally refined equality on sets for code generation
2012-02-02, by bulwahn
adding an example for a datatype refinement which would allow rtrancl to be executable on an infinite type
2012-02-02, by bulwahn
improving code equations for multisets that violated the distinct AList abstraction
2012-02-01, by bulwahn
tuning
2012-02-02, by blanchet
implemented partial application aliases (for SPASS mainly)
2012-02-02, by blanchet
really fixed syntax bug in DFG output (cf. ef62c2fafa9e)
2012-02-01, by blanchet
don't stumble on SPASS debug output
2012-02-01, by blanchet
tuning
2012-02-01, by blanchet
proper statuses for "fact_from_ref"
2012-02-01, by blanchet
tuned
2012-01-31, by nipkow
renamed Sledgehammer option
2012-01-31, by blanchet
third attempt at lambda lifting that works for both Sledgehammer and Metis (cf. dce6c3a460a9)
2012-01-31, by blanchet
improve SPASS setup
2012-01-31, by blanchet
adding code equation for setsum
2012-01-31, by bulwahn
avoid name clash, really
2012-01-31, by blanchet
fixed syntax bug in DFG output
2012-01-31, by blanchet
new SPASS setup
2012-01-31, by blanchet
distinguish between ":lr" and ":lt" (terminating) in DFG format
2012-01-31, by blanchet
nicer keyword class avoidance scheme
2012-01-31, by blanchet
new try at lambda-lifting that works correctly for both Metis and Sledgehammer (cf. d724066ff3d0)
2012-01-31, by blanchet
mutabelle must handle the case where quickcheck returns multiple results
2012-01-31, by bulwahn
reverted e2b1a86d59fc -- broke Metis's lambda-lifting
2012-01-31, by blanchet
merged
2012-01-31, by nipkow
NEWS
2012-01-31, by nipkow
added "'a rel"
2012-01-30, by nipkow
fix debilitating bug with lambda lifting in conjectures with outer existential quantifiers
2012-01-30, by blanchet
new SPASS setup
2012-01-30, by blanchet
example tuning
2012-01-30, by blanchet
implemented new lambda translations scheme
2012-01-30, by blanchet
avoid unsupported case in Metis
2012-01-30, by blanchet
docs and news
2012-01-30, by blanchet
rename lambda translation schemes
2012-01-30, by blanchet
example tuning
2012-01-30, by blanchet
NEWS
2012-01-30, by bulwahn
renaming all lemmas with name rel_pow to relpow
2012-01-30, by bulwahn
adding code equations for max_extp and mlex
2012-01-30, by bulwahn
adding code generation for relpow by copying the ideas for code generation of funpow
2012-01-30, by bulwahn
adding code equation for rtranclp in Enum
2012-01-30, by bulwahn
adding code equation for max_ext
2012-01-30, by bulwahn
adding code equation for tranclp
2012-01-30, by bulwahn
adding code_unfold to make measure executable
2012-01-30, by bulwahn
removed accidental dependance of abstract interpreter on gamma
2012-01-29, by nipkow
merged
2012-01-29, by nipkow
tuned
2012-01-29, by nipkow
an executable version of accessible part (only for finite types yet)
2012-01-28, by bulwahn
adding yet another induction rule on natural numbers
2012-01-28, by bulwahn
moving declarations back to the section they seem to belong to (cf. afffe1f72143)
2012-01-28, by bulwahn
reverting 46c2c96f5d92 as it only provides mostly non-terminating executions for generated code
2012-01-28, by bulwahn
adding some more examples for quickcheck; replaced FIXME comments
2012-01-27, by bulwahn
new code equation for ntrancl that allows computation of the transitive closure of sets on infinite types as well
2012-01-27, by bulwahn
removed duplicate definitions that made locale inconsistent
2012-01-27, by nipkow
added parity analysis
2012-01-27, by nipkow
corrected expectation; added an example for quickcheck
2012-01-27, by bulwahn
adding some basic handling that unfolds a conjecture in a locale before testing it with quickcheck
2012-01-27, by bulwahn
made SML/NJ happy
2012-01-27, by blanchet
even more lr tags for SPASS -- anything that is considered an "equational rule spec" is relevant
2012-01-26, by blanchet
separate orthogonal components
2012-01-26, by blanchet
generate left-to-right rewrite tag for combinator helpers for SPASS 3.8
2012-01-26, by blanchet
better handling of individual type for DFG format (SPASS)
2012-01-26, by blanchet
adding quickcheck example with THE
2012-01-26, by bulwahn
evaluation of THE with a non-singleton set raises a Match exception during the evaluation to yield a potential counterexample in quickcheck.
2012-01-26, by bulwahn
using fully qualified module names in Haskell source, which seems to be required by GHC 7.0.4
2012-01-26, by bulwahn
tuned
2012-01-26, by nipkow
adding very basic code generation to Wellfounded theory
2012-01-25, by bulwahn
removing dead code from Mutabelle; tuned
2012-01-25, by bulwahn
generalizing check if size matters because it is different for random and exhaustive testing
2012-01-25, by bulwahn
merged
2012-01-25, by bulwahn
adding code equation for Collect on finite types
2012-01-25, by bulwahn
Use lookup_size rather than Datatype.get_info in is_poly to avoid
2012-01-24, by berghofe
adding some rules to quickcheck's preprocessing
2012-01-24, by bulwahn
some more constants on mutabelle's blacklist
2012-01-24, by bulwahn
implemented "tptp_refute" tool
2012-01-23, by blanchet
added problem importer
2012-01-23, by blanchet
imported patch ATP_Problem_Import.thy
2012-01-23, by blanchet
imported patch atp_problem_import.ML
2012-01-23, by blanchet
renamed theory exporter
2012-01-23, by blanchet
renamed two files to make room for a new file
2012-01-23, by blanchet
rebranded Nitrox, for more uniformity
2012-01-23, by blanchet
moved "nitrox" to TPTP
2012-01-23, by blanchet
generalize type of List.listrel
2012-01-23, by huffman
support for Ex1 in quickcheck-narrowing
2012-01-23, by bulwahn
adding another internal constant to mutabelle's blacklust
2012-01-23, by bulwahn
adding some more forbidden constant names for the mutated conjecture generation
2012-01-23, by bulwahn
adding code generation for some list relations
2012-01-23, by bulwahn
adding fun_eq_iff to the preprocessing
2012-01-23, by bulwahn
random instance for sets
2012-01-23, by bulwahn
more configurations to mutabelle
2012-01-23, by bulwahn
catching code generation errors in quickcheck-narrowing
2012-01-20, by bulwahn
adding narrowing instance for sets
2012-01-20, by bulwahn
shortened definitions by adding some termify constants
2012-01-20, by bulwahn
tuned
2012-01-20, by bulwahn
adding check_all instance for sets; tuned
2012-01-20, by bulwahn
tuned
2012-01-20, by nipkow
tuned
2012-01-20, by nipkow
minor edits in docs
2012-01-19, by blanchet
renamed "sound" option to "strict"
2012-01-19, by blanchet
updated Sledge docs some more
2012-01-19, by blanchet
more doc updates
2012-01-19, by blanchet
updated docs
2012-01-19, by blanchet
lower timeout for preplay, now that we have more preplay methods
2012-01-19, by blanchet
cleanly separate each Metis encoding
2012-01-19, by blanchet
basic setup for equational reasoning;
2012-02-09, by wenzelm
tuned;
2012-02-07, by wenzelm
updated examples for syntax translations;
2012-02-07, by wenzelm
updated section on raw syntax;
2012-02-05, by wenzelm
updated section about syntax ambiguity;
2012-02-05, by wenzelm
updated/unified section on mixfix annotations;
2012-02-04, by wenzelm
tuned;
2012-02-04, by wenzelm
more on explicit notation;
2012-02-04, by wenzelm
more accurate Pure grammar;
2012-02-04, by wenzelm
more refs;
2012-02-04, by wenzelm
simplified mixfix (NB: infix is no longer required separately);
2012-02-04, by wenzelm
updated section on print modes;
2012-02-02, by wenzelm
misc tuning and reformatting;
2012-02-02, by wenzelm
clarified syntax section structure;
2012-02-02, by wenzelm
discontinued obscure history commands;
2012-02-02, by wenzelm
misc tuning and reformatting;
2012-02-02, by wenzelm
discontinued obscure history commands;
2012-02-02, by wenzelm
updated hint about asm_rl;
2012-01-29, by wenzelm
updated thin_tac;
2012-01-29, by wenzelm
updated distinct_subgoals_tac, flexflex_tac;
2012-01-29, by wenzelm
removed obscure material;
2012-01-29, by wenzelm
updated rotate_tac;
2012-01-29, by wenzelm
tuned;
2012-01-27, by wenzelm
updated citations;
2012-01-27, by wenzelm
updated subgoal_tac;
2012-01-27, by wenzelm
tuned sectioning;
2012-01-26, by wenzelm
updated "Control and search tacticals" (moved from ref to implementation);
2012-01-26, by wenzelm
obsolete -- covered in implementation manual;
2012-01-26, by wenzelm
moved HEADGOAL;
2012-01-26, by wenzelm
removed some obscure material;
2012-01-26, by wenzelm
added SELECT_GOAL;
2012-01-26, by wenzelm
tuned;
2012-01-26, by wenzelm
updated "subgoal quantifiers";
2012-01-25, by wenzelm
tuned ML infixes;
2012-01-25, by wenzelm
document antiquotations for ML infix operators;
2012-01-25, by wenzelm
tuned;
2012-01-25, by wenzelm
updated repetition tacticals;
2012-01-25, by wenzelm
updated THEN, ORELSE, APPEND, and derivatives;
2012-01-25, by wenzelm
removed obscure/outdated material;
2012-01-25, by wenzelm
updated RSN, RL, RLN, MRS;
2012-01-25, by wenzelm
removed obscure/outdated material;
2012-01-25, by wenzelm
tuned;
2012-01-25, by wenzelm
more on Logic.all/mk_implies etc.;
2012-01-25, by wenzelm
reduce AFP test by many hours;
2012-01-19, by wenzelm
added termination of narrowing
2012-01-19, by nipkow
really need 64bit here;
2012-01-18, by wenzelm
Added termination proof for widening
2012-01-18, by nipkow
switch afp test to Darwin on macbroy2
2012-01-18, by kleing
merged
2012-01-18, by nipkow
introduced commands over a set of vars
2012-01-18, by nipkow
basic support for PIDE Scala programming, independently of the main Isabelle repository;
2012-01-18, by wenzelm
fixed a bug introduced when porting functions to set -- extensionality on sets break the form of equations expected elsewhere by Nitpick
2012-01-17, by blanchet
updated message
2012-01-17, by blanchet
improve installation instructions
2012-01-17, by blanchet
allow use of proxy for remote SMT solver invocations, just like in the "remote_atp" script
2012-01-17, by blanchet
factor-cancellation simprocs now call the full simplifier to prove that factors are non-zero
2012-01-17, by huffman
refreshing NEWS
2012-01-17, by bulwahn
renaming theory AList_Impl back to AList (reverting 1fec5b365f9b; AList with distinct key invariant is called DAList)
2012-01-17, by bulwahn
renamed theory AList to DAList
2012-01-17, by bulwahn
position constraints for numerals enable PIDE markup;
2012-01-16, by wenzelm
more careful cumulation of tooltips -- ensure uniform range;
2012-01-16, by wenzelm
tuned;
2012-01-16, by wenzelm
tuned
2012-01-16, by nipkow
missing dependency
2012-01-16, by nipkow
tuned example;
2012-01-15, by wenzelm
merged
2012-01-15, by wenzelm
back to more basic caret_range (reverting 0ad063afa3d6) -- BreakIterator crashes due to non-zero text.offset when deleting the first character of the buffer;
2012-01-15, by wenzelm
recovered outdated_color (cf. 4beb2f41ed93);
2012-01-15, by wenzelm
more precise rendering of overview_color/gutter_message/squiggly_underline based on cumulation of command status and warning/error messages;
2012-01-15, by wenzelm
tuned proofs;
2012-01-15, by wenzelm
tuned
2012-01-15, by nipkow
tuned signature;
2012-01-15, by wenzelm
comments;
2012-01-15, by wenzelm
tuned proofs;
2012-01-15, by wenzelm
eliminated dead code, together with spurious warning about congruence rule for "Fun.comp";
2012-01-15, by wenzelm
more explicit/robust treatment of common snapshot;
2012-01-15, by wenzelm
discontinued old-style Term.list_abs in favour of plain Term.abs;
2012-01-14, by wenzelm
renamed Term.list_all to Logic.list_all, in accordance to HOLogic.list_all;
2012-01-14, by wenzelm
renamed Term.all to Logic.all_const, in accordance to HOLogic.all_const;
2012-01-14, by wenzelm
tuned;
2012-01-14, by wenzelm
discontinued old-style Term.list_all_free in favour of plain Logic.all;
2012-01-14, by wenzelm
tuned;
2012-01-14, by wenzelm
discontinued default rendering for Oheimb's double-space;
2012-01-14, by wenzelm
tuned white space;
2012-01-14, by wenzelm
tuned comment;
2012-01-14, by wenzelm
paranoia null check -- prevent spurious crash of jedit token markup;
2012-01-14, by wenzelm
tuned comments;
2012-01-14, by wenzelm
tuned signature;
2012-01-14, by wenzelm
clarified partial restrict operation;
2012-01-14, by wenzelm
tuned proofs;
2012-01-14, by wenzelm
ignore empty gfx_range;
2012-01-14, by wenzelm
tuned signature;
2012-01-14, by wenzelm
tuned
2012-01-13, by nipkow
handle specific exception, not arbitrary ones (including Interrupt);
2012-01-13, by wenzelm
eliminated dead code;
2012-01-13, by wenzelm
more modest settings for lxbroy10 -- might actually perform better;
2012-01-12, by wenzelm
tuned;
2012-01-12, by wenzelm
improved select_markup: include filtering of defined results;
2012-01-12, by wenzelm
tuned text_color: cumulate with explicit default color;
2012-01-12, by wenzelm
added cat_lines convenience;
2012-01-12, by wenzelm
tuned;
2012-01-12, by wenzelm
clarified mkString: no extra line-breaks for XML.Body;
2012-01-12, by wenzelm
adding exhaustive instances for type constructor set
2012-01-12, by bulwahn
Updated generated file
2012-01-12, by berghofe
Added inf_Int_eq to pred_set_conv database as well
2012-01-12, by berghofe
more conventional eval_tac vs. method_setup "eval";
2012-01-11, by wenzelm
updated generated file -- change of printed case syntax probably due to f805747f8571;
2012-01-11, by wenzelm
actually try to preserve names given by user (cf. 463b594e186a);
2012-01-11, by wenzelm
updated example -- List.foldl is no longer defined via primrec;
2012-01-11, by wenzelm
more qualified names;
2012-01-11, by wenzelm
refer to imp_cong from HOL, not Drule (!) -- cf. 4ed94d92ae19;
2012-01-11, by wenzelm
more robust ISABELLE_HOME_USER for repository versions -- some versions of Emacs interpret foo//bar as /bar even on the command-line (unlike regular POSIX semantics);
2012-01-11, by wenzelm
merged
2012-01-11, by berghofe
Removed strange hack introduced in b27e93132603, since equivariance
2012-01-11, by berghofe
Replaced perm_set_eq by perm_set_def
2012-01-10, by berghofe
Corrected pt_set_inst, added missing cp_set_inst, deleted obsolete
2012-01-10, by berghofe
Reverted several lemmas involving sets to the state before the
2012-01-10, by berghofe
clarified Isabelle_Rendering vs. physical painting;
2012-01-10, by wenzelm
pred_subset_eq and SUP_UN_eq2 are now standard pred_set_conv rules
2012-01-10, by berghofe
pred_subset/equals_eq are now standard pred_set_conv rules
2012-01-10, by berghofe
Declared pred_equals/subset_eq, sup_Un_eq and SUP_UN_eq(2) as pred_set_conv rules
2012-01-10, by berghofe
merged
2012-01-10, by huffman
add simp rules for set_bit and msb applied to 0 and 1
2012-01-10, by huffman
add simp rule test_bit_1
2012-01-10, by huffman
proper hiding of facts and constants in AList_Impl and AList theory
2012-01-10, by bulwahn
NEWS
2012-01-10, by bulwahn
adding quickcheck examples with multisets
2012-01-10, by bulwahn
improving code generation for multisets; adding exhaustive quickcheck generators for multisets
2012-01-10, by bulwahn
adding theory association lists with invariant
2012-01-10, by bulwahn
command status color via regular markup;
2012-01-09, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-512
+512
+1000
+3000
+10000
+30000
tip