Skip to content
GitLab
Menu
Projects
Groups
Snippets
Loading...
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Menu
Open sidebar
isa-afp
afp-devel
Commits
b29f17ffaa83
Commit
ab3ade0d
authored
May 04, 2018
by
immler
Browse files
fixed proofs
parent
85324e3788b7
Changes
3
Hide whitespace changes
Inline
Side-by-side
thys/LLL_Basis_Reduction/LLL_Number_Bounds.thy
View file @
b29f17ff
...
...
@@ -25,9 +25,9 @@ begin
(* TODO: Documentation and add references to computer algebra book *)
hide_const (open) Determinants.det
hide_const (open) Cartesian_
Euclidean_Space
.mat
hide_const (open) Cartesian_
Euclidean_Space
.row
hide_const (open) Cartesian_
Euclidean_Space
.vec
hide_const (open)
Finite_
Cartesian_
Product
.mat
hide_const (open)
Finite_
Cartesian_
Product
.row
hide_const (open)
Finite_
Cartesian_
Product
.vec
hide_const (open) Path_Connected.outside
hide_const (open) Linear_Algebra.orthogonal
hide_type (open) Finite_Cartesian_Product.vec
...
...
thys/LLL_Basis_Reduction/Missing_Lemmas.thy
View file @
b29f17ff
...
...
@@ -1612,7 +1612,7 @@ lemma mem_set_find_indices [simp]: "i \<in> set (find_indices x xs) \<longleftri
lemma distinct_find_indices: "distinct (find_indices x xs)"
unfolding find_indices_def by simp
context module begin
context
Module.
module begin
definition lincomb_list
where "lincomb_list c vs = sumlist (map (\<lambda>i. c i \<odot>\<^bsub>M\<^esub> vs ! i) [0..<length vs])"
...
...
thys/Ordinary_Differential_Equations/Numerics/Example_Utilities.thy
View file @
b29f17ff
...
...
@@ -1013,9 +1013,7 @@ lemma blinfuns_of_lvivl_eq: "blinfuns_of_lvivl x =
lemma range_blinfun_of_vmatrix[simp]: "range blinfun_of_vmatrix = UNIV"
apply auto
apply transfer
subgoal for x
unfolding linear_linear
by (auto intro!: matrix_works[symmetric])
subgoal for x by (rule image_eqI[where x="matrix x"]) auto
done
lemma blinfun_of_vmatrix_image:
...
...
Write
Preview
Markdown
is supported
0%
Try again
or
attach a new file
.
Attach a file
Cancel
You are about to add
0
people
to the discussion. Proceed with caution.
Finish editing this message first!
Cancel
Please
register
or
sign in
to comment